Skip to content

Commit 1aece6a

Browse files
committed
test fix
1 parent 31b7c6a commit 1aece6a

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

test/LawfulOrd.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -13,7 +13,7 @@ nLtEq2Gt : ⦃ iOrdA : Ord a ⦄ → ⦃ IsLawfulOrd a ⦄
1313
nLtEq2Gt x y ⦃ h1 ⦄ ⦃ h2 ⦄ =
1414
begin
1515
(x > y)
16-
≡⟨ sym (not-involution (x <= y) (x > y) (lte2ngt x y)) ⟩
16+
≡⟨ sym (not-involution (lte2ngt x y)) ⟩
1717
not (x <= y)
1818
≡⟨ cong not (lte2LtEq x y) ⟩
1919
not ((x < y) || (x == y))

0 commit comments

Comments
 (0)