@@ -21,6 +21,10 @@ Bug-fixes
21
21
* The binary relation ` _≉_ ` exposed by records in ` Relation.Binary.Bundles ` now has
22
22
the correct infix precedence.
23
23
24
+ * Fixed the fixity of the reasoning combinators in
25
+ ` Data.List.Relation.Binary.Subset.(Propositional/Setoid).Properties ` so that they
26
+ compose properly.
27
+
24
28
* Added version to library name
25
29
26
30
Non-backwards compatible changes
@@ -33,24 +37,28 @@ Non-backwards compatible changes
33
37
* The module ` Algebra.Construct.Zero ` and ` Algebra.Module.Construct.Zero `
34
38
are now level-polymorphic, each taking two implicit level parameters.
35
39
36
- * Previously the definition of ` _⊖_ ` in ` Data.Integer.Base ` was defined
37
- inductively as:
40
+ * Previously ` _⊖_ ` in ` Data.Integer.Base ` was defined inductively as:
38
41
``` agda
39
42
_⊖_ : ℕ → ℕ → ℤ
40
43
m ⊖ ℕ.zero = + m
41
44
ℕ.zero ⊖ ℕ.suc n = -[1+ n ]
42
45
ℕ.suc m ⊖ ℕ.suc n = m ⊖ n
43
46
```
44
- which meant that the unary arguments had to be evaluated. To make it
45
- much faster it's definition has been changed to use operations on ` ℕ `
46
- that are backed by builtin operations:
47
+ which meant that it had to recursively evaluate its unary arguments.
48
+ The definition has been changed as follows to use operations on ` ℕ ` that are backed
49
+ by builtin operations, greatly improving its performance :
47
50
``` agda
48
51
_⊖_ : ℕ → ℕ → ℤ
49
52
m ⊖ n with m ℕ.<ᵇ n
50
53
... | true = - + (n ℕ.∸ m)
51
54
... | false = + (m ℕ.∸ n)
52
55
```
53
56
57
+ * The proofs ` ↭⇒∼bag ` and ` ∼bag⇒↭ ` have been moved from
58
+ ` Data.List.Relation.Binary.Permutation.Setoid.Properties `
59
+ to ` Data.List.Relation.Binary.BagAndSetEquality ` as their current location
60
+ were causing cyclic import dependencies.
61
+
54
62
Deprecated modules
55
63
------------------
56
64
@@ -97,6 +105,24 @@ Deprecated names
97
105
Plus′ ↦ TransClosure
98
106
```
99
107
108
+ * In ` Data.List.Relation.Binary.Subset.Propositional.Properties ` :
109
+ ``` agda
110
+ mono ↦ Any-resp-⊆
111
+ map-mono ↦ map⁺
112
+ concat-mono ↦ concat⁺
113
+ >>=-mono ↦ >>=⁺
114
+ _⊛-mono_ ↦ ⊛⁺
115
+ _⊗-mono_ ↦ ⊗⁺
116
+ any-mono ↦ any⁺
117
+ map-with-∈-mono ↦ map-with-∈⁺
118
+ filter⁺ ↦ filter-⊆
119
+ ```
120
+
121
+ * In ` Data.List.Relation.Binary.Subset.Setoid.Properties ` :
122
+ ``` agda
123
+ filter⁺ ↦ filter-⊆
124
+ ```
125
+
100
126
New modules
101
127
-----------
102
128
@@ -236,6 +262,60 @@ Other minor additions
236
262
m-n≡m⊖n : + m + (- + n) ≡ m ⊖ n
237
263
```
238
264
265
+ * Added new relations in ` Data.List.Relation.Binary.Subset.(Propositional/Setoid) ` :
266
+ ``` agda
267
+ xs ⊇ ys = ys ⊆ xs
268
+ xs ⊉ ys = ¬ xs ⊇ ys
269
+ ```
270
+
271
+ * Added new proofs in ` Data.List.Relation.Binary.Subset.Propositional.Properties ` :
272
+ ``` agda
273
+ ⊆-respʳ-≋ : _⊆_ Respectsʳ _≋_
274
+ ⊆-respˡ-≋ : _⊆_ Respectsˡ _≋_
275
+
276
+ ↭⇒⊆ : _↭_ ⇒ _⊆_
277
+ ⊆-respʳ-↭ : _⊆_ Respectsʳ _↭_
278
+ ⊆-respˡ-↭ : _⊆_ Respectsˡ _↭_
279
+ ⊆-↭-isPreorder : IsPreorder _↭_ _⊆_
280
+ ⊆-↭-preorder : Preorder _ _ _
281
+
282
+ Any-resp-⊆ : P Respects _≈_ → (Any P) Respects _⊆_
283
+ All-resp-⊇ : P Respects _≈_ → (All P) Respects _⊇_
284
+
285
+ xs⊆xs++ys : xs ⊆ xs ++ ys
286
+ xs⊆ys++xs : xs ⊆ ys ++ xs
287
+ ++⁺ʳ : xs ⊆ ys → zs ++ xs ⊆ zs ++ ys
288
+ ++⁺ˡ : xs ⊆ ys → xs ++ zs ⊆ ys ++ zs
289
+ ++⁺ : ws ⊆ xs → ys ⊆ zs → ws ++ ys ⊆ xs ++ zs
290
+ ```
291
+
292
+ * Added new proofs in ` Data.List.Relation.Binary.Subset.Propositional.Properties ` :
293
+ ``` agda
294
+ ↭⇒⊆ : _↭_ ⇒ _⊆_
295
+ ⊆-respʳ-↭ : _⊆_ Respectsʳ _↭_
296
+ ⊆-respˡ-↭ : _⊆_ Respectsˡ _↭_
297
+ ⊆-↭-isPreorder : IsPreorder _↭_ _⊆_
298
+ ⊆-↭-preorder : Preorder _ _ _
299
+
300
+ Any-resp-⊆ : (Any P) Respects _⊆_
301
+ All-resp-⊇ : (All P) Respects _⊇_
302
+
303
+ xs⊆xs++ys : xs ⊆ xs ++ ys
304
+ xs⊆ys++xs : xs ⊆ ys ++ xs
305
+ ++⁺ʳ : xs ⊆ ys → zs ++ xs ⊆ zs ++ ys
306
+ ++⁺ˡ : xs ⊆ ys → xs ++ zs ⊆ ys ++ zs
307
+ ```
308
+
309
+ * Added new proof in ` Data.List.Relation.Binary.Permutation.Propositional.Properties ` :
310
+ ``` agda
311
+ ++↭ʳ++ : xs ++ ys ↭ xs ʳ++ ys
312
+ ```
313
+
314
+ * Added new proof in ` Data.List.Relation.Binary.Permutation.Setoi.Properties ` :
315
+ ``` agda
316
+ ++↭ʳ++ : xs ++ ys ↭ xs ʳ++ ys
317
+ ```
318
+
239
319
* Added new definition in ` Data.Nat.Base ` :
240
320
``` agda
241
321
_≤ᵇ_ : (m n : ℕ) → Bool
0 commit comments