Skip to content

Commit

Permalink
Int cleanup
Browse files Browse the repository at this point in the history
  • Loading branch information
odderwiser committed Dec 9, 2024
1 parent 6ab31b8 commit 7c1d356
Showing 1 changed file with 0 additions and 7 deletions.
7 changes: 0 additions & 7 deletions lib/Haskell/Law/Ord/Int.agda
Original file line number Diff line number Diff line change
Expand Up @@ -13,13 +13,6 @@ open import Haskell.Law.Eq
open import Haskell.Law.Ord.Def
open import Haskell.Law.Int

private

2⁶³ : Nat
2⁶³ = 9223372036854775808

maxW : Word
maxW = (n2w (monusNat 2⁶³ 1))

sign2neq : (a b : Int) isNegativeInt a ≡ True isNegativeInt b ≡ False ((a == b) ≡ False)
sign2neq a@(int64 x) b@(int64 y) h₁ h₂ with a == b in h₃
Expand Down

0 comments on commit 7c1d356

Please sign in to comment.