File tree Expand file tree Collapse file tree 3 files changed +116
-73
lines changed Expand file tree Collapse file tree 3 files changed +116
-73
lines changed Original file line number Diff line number Diff line change @@ -235,6 +235,17 @@ Backwards compatible changes
235
235
∩⇔× : x ∈ p ∩ q ⇔ (x ∈ p × x ∈ q)
236
236
```
237
237
238
+ * Added relations to ` Data.Integer `
239
+ ``` agda
240
+ _≥_ : Rel ℤ _
241
+ _<_ : Rel ℤ _
242
+ _>_ : Rel ℤ _
243
+ _≰_ : Rel ℤ _
244
+ _≱_ : Rel ℤ _
245
+ _≮_ : Rel ℤ _
246
+ _≯_ : Rel ℤ _
247
+ ```
248
+
238
249
* Added proofs to ` Data.Integer.Properties `
239
250
``` agda
240
251
+-injective : + m ≡ + n → m ≡ n
@@ -260,6 +271,7 @@ Backwards compatible changes
260
271
+-inverse : Inverse (+ 0) -_ _+_
261
272
+-0-isMonoid : IsMonoid _≡_ _+_ (+ 0)
262
273
+-0-isGroup : IsGroup _≡_ _+_ (+ 0) (-_)
274
+ +-0-abelianGroup : AbelianGroup _ _
263
275
neg-distrib-+ : - (m + n) ≡ (- m) + (- n)
264
276
◃-distrib-+ : s ◃ (m + n) ≡ (s ◃ m) + (s ◃ n)
265
277
Original file line number Diff line number Diff line change @@ -18,7 +18,7 @@ open import Relation.Binary.Core using (_≡_; refl)
18
18
infix 8 -_
19
19
infixl 7 _*_ _⊓_
20
20
infixl 6 _+_ _-_ _⊖_ _⊔_
21
- infix 4 _≤_
21
+ infix 4 _≤_ _≥_ _<_ _>_ _≰_ _≱_ _≮_ _≯_
22
22
23
23
------------------------------------------------------------------------
24
24
-- The types
@@ -149,6 +149,27 @@ data _≤_ : ℤ → ℤ → Set where
149
149
-≤- : ∀ {m n} → (n≤m : n ℕ.≤ m) → -[1+ m ] ≤ -[1+ n ]
150
150
+≤+ : ∀ {m n} → (m≤n : m ℕ.≤ n) → + m ≤ + n
151
151
152
+ _≥_ : Rel ℤ _
153
+ x ≥ y = y ≤ x
154
+
155
+ _<_ : Rel ℤ _
156
+ x < y = suc x ≤ y
157
+
158
+ _>_ : Rel ℤ _
159
+ x > y = y < x
160
+
161
+ _≰_ : Rel ℤ _
162
+ x ≰ y = ¬ (x ≤ y)
163
+
164
+ _≱_ : Rel ℤ _
165
+ x ≱ y = ¬ (x ≥ y)
166
+
167
+ _≮_ : Rel ℤ _
168
+ x ≮ y = ¬ (x < y)
169
+
170
+ _≯_ : Rel ℤ _
171
+ x ≯ y = ¬ (x > y)
172
+
152
173
drop‿+≤+ : ∀ {m n} → + m ≤ + n → ℕ._≤_ m n
153
174
drop‿+≤+ (+≤+ m≤n) = m≤n
154
175
You can’t perform that action at this time.
0 commit comments