Skip to content

Commit

Permalink
test fix
Browse files Browse the repository at this point in the history
  • Loading branch information
odderwiser committed Dec 9, 2024
1 parent 31b7c6a commit 1aece6a
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion test/LawfulOrd.agda
Original file line number Diff line number Diff line change
Expand Up @@ -13,7 +13,7 @@ nLtEq2Gt : ⦃ iOrdA : Ord a ⦄ → ⦃ IsLawfulOrd a ⦄
nLtEq2Gt x y ⦃ h1 ⦄ ⦃ h2 ⦄ =
begin
(x > y)
≡⟨ sym (not-involution (x <= y) (x > y) (lte2ngt x y)) ⟩
≡⟨ sym (not-involution (lte2ngt x y)) ⟩
not (x <= y)
≡⟨ cong not (lte2LtEq x y) ⟩
not ((x < y) || (x == y))
Expand Down

0 comments on commit 1aece6a

Please sign in to comment.