Skip to content

Commit

Permalink
Eq Double removal
Browse files Browse the repository at this point in the history
  • Loading branch information
odderwiser authored and jespercockx committed Feb 27, 2024
1 parent 3ab718a commit c4b26e2
Showing 1 changed file with 0 additions and 2 deletions.
2 changes: 0 additions & 2 deletions lib/Haskell/Law/Eq/Def.agda
Original file line number Diff line number Diff line change
Expand Up @@ -66,5 +66,3 @@ eqNegation : ⦃ iEq : Eq e ⦄ → ⦃ IsLawfulEq e ⦄
{ x y : e } (x /= y) ≡ not (x == y)
eqNegation = refl

postulate instance
iLawfulEqDouble : IsLawfulEq Double

0 comments on commit c4b26e2

Please sign in to comment.