You signed in with another tab or window. Reload to refresh your session.You signed out in another tab or window. Reload to refresh your session.You switched accounts on another tab or window. Reload to refresh your session.Dismiss alert
Copy file name to clipboardExpand all lines: src/Data/Integer/IntConstruction/Properties.agda
+62Lines changed: 62 additions & 0 deletions
Original file line number
Diff line number
Diff line change
@@ -12,6 +12,7 @@ import Algebra.Properties.CommutativeSemigroup as CommSemigroupProps
12
12
open importData.Integer.IntConstruction
13
13
open importData.Nat.Base as ℕ using (ℕ)
14
14
importData.Nat.Properties as ℕ
15
+
open importData.Product.Base
15
16
open importFunction.Base
16
17
open importRelation.Binary
17
18
open importRelation.Binary.PropositionalEquality
@@ -62,6 +63,9 @@ _≃?_ : Decidable _≃_
62
63
≤-refl : Reflexive _≤_
63
64
≤-refl = ℕ.≤-refl
64
65
66
+
≤-reflexive : _≃_ ⇒ _≤_
67
+
≤-reflexive = ℕ.≤-reflexive
68
+
65
69
≤-trans : Transitive _≤_
66
70
≤-trans {a ⊖ b} {c ⊖ d} {e ⊖ f} i≤j j≤k = ℕ.+-cancelʳ-≤ (d ℕ.+ c) (a ℕ.+ f) (e ℕ.+ b) $ trans-helper ℕ._≤_ a b c d e f (ℕ.+-mono-≤ i≤j j≤k)
67
71
@@ -253,3 +257,61 @@ _<?_ : Decidable _<_
253
257
254
258
*-comm : Commutative _*_
255
259
*-comm (a ⊖ b) (c ⊖ d) = cong₂ ℕ._+_ (cong₂ ℕ._+_ (ℕ.*-comm a c) (ℕ.*-comm b d)) (trans (ℕ.+-comm (c ℕ.* b) (d ℕ.* a)) (cong₂ ℕ._+_ (ℕ.*-comm d a) (ℕ.*-comm c b)))
0 commit comments