@@ -128,6 +128,19 @@ New modules
128
128
Data.Container.Indexed.Relation.Binary.Equality.Setoid
129
129
```
130
130
131
+ * ` System.Random ` bindings:
132
+ ``` agda
133
+ System.Random.Primitive
134
+ System.Random
135
+ ```
136
+
137
+ * Show modules:
138
+ ``` agda
139
+ Data.List.Show
140
+ Data.Vec.Show
141
+ Data.Vec.Bounded.Show
142
+ ```
143
+
131
144
Additions to existing modules
132
145
-----------------------------
133
146
@@ -252,6 +265,12 @@ Additions to existing modules
252
265
x \\ y = (x ⁻¹) ∙ y
253
266
```
254
267
268
+ * In ` Algebra.Structures.IsCancellativeCommutativeSemiring ` add the
269
+ extra property as an exposed definition:
270
+ ``` agda
271
+ *-cancelʳ-nonZero : AlmostRightCancellative 0# *
272
+ ```
273
+
255
274
* In ` Data.Container.Indexed.Core ` :
256
275
``` agda
257
276
Subtrees o c = (r : Response c) → X (next c r)
@@ -262,6 +281,11 @@ Additions to existing modules
262
281
nonZeroIndex : Fin n → ℕ.NonZero n
263
282
```
264
283
284
+ * In ` Data.Float.Base ` :
285
+ ``` agda
286
+ _≤_ : Rel Float _
287
+ ```
288
+
265
289
* In ` Data.Integer.Divisibility ` : introduce ` divides ` as an explicit pattern synonym
266
290
``` agda
267
291
pattern divides k eq = Data.Nat.Divisibility.divides k eq
@@ -276,6 +300,7 @@ Additions to existing modules
276
300
277
301
* In ` Data.List.Properties ` :
278
302
``` agda
303
+ length-catMaybes : length (catMaybes xs) ≤ length xs
279
304
applyUpTo-∷ʳ : applyUpTo f n ∷ʳ f n ≡ applyUpTo f (suc n)
280
305
applyDownFrom-∷ʳ : applyDownFrom (f ∘ suc) n ∷ʳ f 0 ≡ applyDownFrom f (suc n)
281
306
upTo-∷ʳ : upTo n ∷ʳ n ≡ upTo (suc n)
@@ -409,6 +434,13 @@ Additions to existing modules
409
434
* Added new functions in ` Data.String.Base ` :
410
435
``` agda
411
436
map : (Char → Char) → String → String
437
+ between : String → String → String → String
438
+ ```
439
+
440
+ * In ` Data.Word.Base ` :
441
+ ``` agda
442
+ _≤_ : Rel Word64 zero
443
+ ```
412
444
413
445
* Added new definition in ` Relation.Binary.Construct.Closure.Transitive `
414
446
```
@@ -457,5 +489,7 @@ Additions to existing modules
457
489
WeaklyDecidable : Pred A ℓ → Set _
458
490
```
459
491
460
- * ` Tactic.Cong ` now provides a marker function, ` ⌞_⌟ ` , for user-guided
461
- anti-unification. See README.Tactic.Cong for details.
492
+ * Enhancements to ` Tactic.Cong ` - see ` README.Tactic.Cong ` for details.
493
+ - Provide a marker function, ` ⌞_⌟ ` , for user-guided anti-unification.
494
+ - Improved support for equalities between terms with instance arguments,
495
+ such as terms that contain ` _/_ ` or ` _%_ ` .
0 commit comments