05-equality-std2.agda 672 B

12345678910111213141516171819202122232425
  1. {-# OPTIONS --universe-polymorphism #-}
  2. -- {-# OPTIONS --verbose tc.rec:15 #-}
  3. -- {-# OPTIONS --verbose tc.records.ifs:15 #-}
  4. -- {-# OPTIONS --verbose tc.constr.findInScope:15 #-}
  5. -- {-# OPTIONS --verbose tc.term.args.ifs:15 #-}
  6. module InstanceArguments.05-equality-std2 where
  7. open import Agda.Primitive
  8. open import Relation.Nullary
  9. open import Relation.Binary
  10. open import Relation.Binary.PropositionalEquality using (_≡_)
  11. open import Data.Bool hiding (_≟_)
  12. open import Data.Bool.Properties using (≡-decSetoid)
  13. open DecSetoid {{...}}
  14. instance
  15. decBool = ≡-decSetoid
  16. test : IsDecEquivalence (_≡_ {A = Bool})
  17. test = isDecEquivalence
  18. test2 = false ≟ false