EqReasoning.agda 325 B

123456789101112131415161718192021
  1. open import Data.Nat.Base
  2. open import Relation.Binary.PropositionalEquality
  3. open ≡-Reasoning
  4. test : 0 ≡ 0
  5. test = begin
  6. 0 ≡⟨ {!!} ⟩
  7. 0
  8. -- WAS: Goal is garbled:
  9. --
  10. -- ?0 : (.Relation.Binary.Setoid.preorder (setoid ℕ)
  11. -- .Relation.Binary.Preorder.∼ 0)
  12. -- 0
  13. -- EXPECTED: Nice goal:
  14. --
  15. -- ?0 : 0 ≡ 0