We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent 31b7c6a commit 1aece6aCopy full SHA for 1aece6a
test/LawfulOrd.agda
@@ -13,7 +13,7 @@ nLtEq2Gt : ⦃ iOrdA : Ord a ⦄ → ⦃ IsLawfulOrd a ⦄
13
nLtEq2Gt x y ⦃ h1 ⦄ ⦃ h2 ⦄ =
14
begin
15
(x > y)
16
- ≡⟨ sym (not-involution (x <= y) (x > y) (lte2ngt x y)) ⟩
+ ≡⟨ sym (not-involution (lte2ngt x y)) ⟩
17
not (x <= y)
18
≡⟨ cong not (lte2LtEq x y) ⟩
19
not ((x < y) || (x == y))
0 commit comments