@@ -21,24 +21,23 @@ Bug-fixes
21
21
* Fixed various algebraic bundles not correctly re-exporting
22
22
` commutativeSemigroup ` proofs.
23
23
24
- * Fix in ` Induction.WellFounded.FixPoint ` , where the well-founded relation ` _<_ ` and
24
+ * Fixed bug in ` Induction.WellFounded.FixPoint ` , where the well-founded relation ` _<_ ` and
25
25
the predicate ` P ` were required to live at the same universe level.
26
26
27
27
Non-backwards compatible changes
28
28
--------------------------------
29
29
30
30
#### Changes to the ` Relation.Unary.Closure ` hierarchy
31
31
32
- * Following the study of the closure operator ` ◇ ` dual to the ` □ ` we originally
33
- provided, the set of modules has been reorganised. We have
32
+ * Following the study of the closure operator ` ◇ ` dual to the ` □ ` operator
33
+ originally provided, the ` Relation.Unary.Closure ` modules have been reorganised.
34
+ We have
34
35
35
36
+ Added the ` ◇ ` closure operator to ` .Base `
36
- + Moved all of the ` □ ` -related functions in submodules called ` □ `
37
- + Added all of the corresponding ` ◇ ` -related functions in submodules called ` ◇ `
38
-
39
- * We also provide functions converting back and forth between ` □ ` -based and
40
- ` ◇ ` -based statements in ` .Base ` :
37
+ + Moved all of the ` □ ` -related functions into submodules called ` □ ` (e.g. ` reindex ` → ` □.reindex ` )
38
+ + Added all of the corresponding ` ◇ ` -related functions into submodules called ` ◇ ` (e.g. ` ◇-reindex ` )
41
39
40
+ * Added functions converting back and forth between ` □ ` -based and ` ◇ ` -based statements in ` .Base ` :
42
41
``` agda
43
42
curry : (∀ {x} → ◇ T x → P x) → (∀ {x} → T x → □ P x)
44
43
uncurry : (∀ {x} → T x → □ P x) → (∀ {x} → ◇ T x → P x)
@@ -48,31 +47,34 @@ Non-backwards compatible changes
48
47
49
48
* The ` n ` argument to ` _⊜_ ` in ` Tactic.RingSolver.NonReflective ` has been made implict rather than explicit.
50
49
51
- * ` Data.Empty.Polymorphic ` and ` Data.Unit.Polymorphic ` were rewritten
52
- to explicitly use ` Lift ` rather that defining new types. This means
53
- that these are now compatible with ` ⊥ ` and ` ⊤ ` from the rest of the
54
- library. This allowed them to be used in the rest of library where
55
- explicit ` Lift ` was used.
50
+ * Made the first argument of ` [,]-∘-distr ` in ` Data.Sum.Properties ` explicit rather than implicit.
51
+
52
+ * ` Data.Empty.Polymorphic ` and ` Data.Unit.Polymorphic ` have been redefined using
53
+ ` Lift ` and the original non-polymorphic versions, rather than being defined as new types. This means
54
+ that these are now compatible with ` ⊥ ` and ` ⊤ ` from the rest of the library,
55
+ allowing them to be used where previously ` Lift ` was used explicitly.
56
56
57
57
Deprecated modules
58
58
------------------
59
59
60
- * ` Data.AVL ` and all of its submodules have been moved to ` Data.Tree.AVL `
61
-
62
60
* The module ` Induction.WellFounded.InverseImage ` has been deprecated. The proofs
63
61
` accessible ` and ` wellFounded ` have been moved to ` Relation.Binary.Construct.On ` .
64
62
65
- * ` Reflection.TypeChecking.MonadSyntax ` ↦ ` Reflection.TypeChecking.Monad.Syntax `
63
+ * The module ` Data.AVL ` and all of its submodules have been renamed to ` Data.Tree.AVL ` .
64
+
65
+ * The module ` Reflection.TypeChecking.MonadSyntax ` has been renamed to
66
+ ` Reflection.TypeChecking.Monad.Syntax ` .
66
67
67
68
Deprecated names
68
69
----------------
69
70
70
71
* The proofs ` replace-equality ` from ` Algebra.Properties.(Lattice/DistributiveLattice/BooleanAlgebra) `
71
72
have been deprecated in favour of the proofs in the new ` Algebra.Construct.Subst.Equality ` module.
72
73
73
- * In order to be consistent in usage of \prime character and apostrophe in identifiers, the following three names were deprecated in favor of their replacement that ends with a \prime character.
74
- * ` Data.List.Base.InitLast._∷ʳ'_ ` ↦ ` Data.List.Base.InitLast._∷ʳ′_ `
75
- * ` Data.List.NonEmpty.SnocView._∷ʳ'_ ` ↦ ` Data.List.NonEmpty.SnocView._∷ʳ′_ `
74
+ * In order to be consistent in usage of \prime character and apostrophe in identifiers,
75
+ the following three names were deprecated in favor of their replacement that ends with a ` \prime ` character.
76
+ * ` Data.List.Base.InitLast._∷ʳ'_ ` ↦ ` Data.List.Base.InitLast._∷ʳ′_ `
77
+ * ` Data.List.NonEmpty.SnocView._∷ʳ'_ ` ↦ ` Data.List.NonEmpty.SnocView._∷ʳ′_ `
76
78
* ` Relation.Binary.Construct.StrictToNonStrict.decidable' ` ↦ ` Relation.Binary.Construct.StrictToNonStrict.decidable′ `
77
79
78
80
* In ` Algebra.Morphism.Definitions ` and ` Relation.Binary.Morphism.Definitions `
@@ -95,15 +97,19 @@ Deprecated names
95
97
*-+-commutativeSemiring ↦ +-*-commutativeSemiring
96
98
*-+-isSemiringWithoutAnnihilatingZero ↦ +-*-isSemiringWithoutAnnihilatingZero
97
99
```
98
- * In ̀Function.Basè:
100
+
101
+ * In ` Function.Base ` :
99
102
```
100
103
*_-[_]-_ ↦ _-⟪_⟫-_
101
104
```
102
105
103
- * ` Data.List.Relation.Unary.Any.any ` to ` Data.List.Relation.Unary.Any.any? `
104
- * ` Data.List.Relation.Unary.All.all ` to ` Data.List.Relation.Unary.All.all? `
105
- * ` Data.Vec.Relation.Unary.Any.any ` to ` Data.Vec.Relation.Unary.Any.any? `
106
- * ` Data.Vec.Relation.Unary.All.all ` to ` Data.Vec.Relation.Unary.All.all? `
106
+ * In ` Data.List.Relation.Unary.Any ` : ` any ↦ any? `
107
+
108
+ * In ` Data.List.Relation.Unary.All ` : ` all ↦ all? `
109
+
110
+ * In ` Data.Vec.Relation.Unary.Any ` ` any ↦ any? `
111
+
112
+ * In ` Data.Vec.Relation.Unary.All ` ` all ↦ all? `
107
113
108
114
New modules
109
115
-----------
@@ -115,7 +121,7 @@ New modules
115
121
Algebra.Module.Construct.DirectProduct.agda
116
122
```
117
123
118
- * Substituting the notion of equality for various structures
124
+ * Substituting the notion of equality for various structures:
119
125
```
120
126
Algebra.Construct.Subst.Equality
121
127
Relation.Binary.Construct.Subst.Equality
@@ -133,7 +139,7 @@ New modules
133
139
Function.Identity.Instances
134
140
```
135
141
136
- * Predicate for lists that are sorted with respect to a total order
142
+ * Predicate for lists that are sorted with respect to a total order:
137
143
```
138
144
Data.List.Relation.Unary.Sorted.TotalOrder
139
145
Data.List.Relation.Unary.Sorted.TotalOrder.Properties
@@ -144,13 +150,13 @@ New modules
144
150
Data.Nat.Binary.Subtraction
145
151
```
146
152
147
- * A predicate for vectors in which every pair of elements is related.
153
+ * A predicate for vectors in which every pair of elements is related:
148
154
```
149
155
Data.Vec.Relation.Unary.AllPairs
150
156
Data.Vec.Relation.Unary.AllPairs.Properties
151
157
```
152
158
153
- * A predicate for vectors in which every element is unique.
159
+ * A predicate for vectors in which every element is unique:
154
160
```
155
161
Data.Vec.Relation.Unary.Unique.Propositional
156
162
Data.Vec.Relation.Unary.Unique.Propositional.Properties
@@ -171,7 +177,7 @@ New modules
171
177
```
172
178
173
179
* Modules replacing ` Function.Related.TypeIsomorphisms ` using the new
174
- ` Inverse ` definitions.
180
+ ` Inverse ` definitions:
175
181
```
176
182
Data.Sum.Algebra
177
183
Data.Product.Algebra
@@ -182,12 +188,12 @@ New modules
182
188
Function.Properties
183
189
```
184
190
185
- * Symmetry for various functional properties
191
+ * Symmetry for various functional properties:
186
192
``` agda
187
193
Function.Construct.Symmetry
188
194
```
189
195
190
- * Added a hierarchy for metric spaces:
196
+ * A hierarchy for metric spaces:
191
197
```
192
198
Function.Metric
193
199
Function.Metric.Core
@@ -206,7 +212,7 @@ New modules
206
212
```
207
213
and other specialisations can be created in a similar fashion.
208
214
209
- * Type -checking monads
215
+ * The type -checking monads:
210
216
```
211
217
Reflection.TypeChecking.Monad
212
218
Reflection.TypeChecking.Monad.Categorical
@@ -230,7 +236,7 @@ New modules
230
236
Relation.Binary.Construct.Composition
231
237
```
232
238
233
- * Generic printf
239
+ * Generic ` printf ` method:
234
240
```
235
241
Text.Format.Generic
236
242
Text.Printf.Generic
@@ -239,25 +245,24 @@ New modules
239
245
Other major changes
240
246
-------------------
241
247
242
- * The module ` Relation.Binary.PropositionalEquality ` has been growing in size and
243
- now depends on a lot of other parts of the library, even though its basic
244
- functionality does not. To fix this some of its parts have been factored out.
245
- ` Relation.Binary.PropositionalEquality.Core ` already existed. Added are:
248
+ * The module ` Relation.Binary.PropositionalEquality ` has recently grown in size and
249
+ now depends on a lot of other parts of the library, e.g. the ` Algebra ` hierarchy,
250
+ even though its basic functionality does not. To allow users the options of avoiding
251
+ specific dependencies, some parts of ` Relation.Binary.PropositionalEquality ` have
252
+ been refactored out into:
246
253
``` agda
247
254
Relation.Binary.PropositionalEquality.Properties
248
255
Relation.Binary.PropositionalEquality.Algebra
249
256
```
250
257
These new modules are re-exported by ` Relation.Binary.PropositionalEquality `
251
- and so these changes should be invisble to current users, but can be useful
252
- to authors of large libraries.
258
+ and so these changes should be invisble to current users.
253
259
254
260
Other minor additions
255
261
---------------------
256
262
257
263
* Add proof to ` Algebra.Morphism.RingMonomorphism ` :
258
264
``` agda
259
- isCommutativeRing : IsCommutativeRing _≈₂_ _⊕_ _⊛_ ⊝_ 0#₂ 1#₂ →
260
- IsCommutativeRing _≈₁_ _+_ _*_ -_ 0# 1#
265
+ isCommutativeRing : IsCommutativeRing _≈₂_ _⊕_ _⊛_ ⊝_ 0#₂ 1#₂ → IsCommutativeRing _≈₁_ _+_ _*_ -_ 0# 1#
261
266
```
262
267
263
268
* Added new proof to ` Data.Fin.Induction ` :
@@ -269,7 +274,7 @@ Other minor additions
269
274
``` agda
270
275
toℕ≤n : (i : Fin n) → toℕ i ≤ n
271
276
≤fromℕ : (i : Fin (suc n)) → i ≤ fromℕ n
272
- fromℕ<-irrelevant : m ≡ n → fromℕ< m<o ≡ fromℕ< n<o
277
+ fromℕ<-cong : m ≡ n → fromℕ< m<o ≡ fromℕ< n<o
273
278
fromℕ<-injective : fromℕ< m<o ≡ fromℕ< n<o → m ≡ n
274
279
inject₁ℕ< : (i : Fin n) → toℕ (inject₁ i) < n
275
280
inject₁ℕ≤ : (i : Fin n) → toℕ (inject₁ i) ≤ n
@@ -455,12 +460,9 @@ Other minor additions
455
460
assocʳ′ : (A × B) × C → A × (B × C)
456
461
assocˡ′ : A × (B × C) → (A × B) × C
457
462
458
- dmap : (f : (a : A) → B a) → (∀ {a} (p : P a) → Q p (f a)) →
459
- (ap : Σ A P) → Σ (B (proj₁ ap)) (Q (proj₂ ap))
460
- dmap : ((a : A) → X a) → ((b : B) → Y b) →
461
- (ab : A × B) → X (proj₁ ab) × Y (proj₂ ab)
462
- _<*>_ : ((a : A) → X a) × ((b : B) → Y b) →
463
- ((a , b) : A × B) → X a × Y b
463
+ dmap : (f : (a : A) → B a) → (∀ {a} (b : P a) → Q b (f a)) → ((a , b) : Σ A P) → Σ (B a) (Q b)
464
+ dmap′ : ((a : A) → X a) → ((b : B) → Y b) → ((a , b) : A × B) → X a × Y b
465
+ _<*>_ : ((a : A) → X a) × ((b : B) → Y b) → ((a , b) : A × B) → X a × Y b
464
466
```
465
467
466
468
* Added new proofs to ` Data.Product.Properties ` :
@@ -476,8 +478,6 @@ Other minor additions
476
478
assocˡ : A ⊎ B ⊎ C → (A ⊎ B) ⊎ C
477
479
```
478
480
479
- * Made first argument of ` [,]-∘-distr ` in ` Data.Sum.Properties ` explicit
480
-
481
481
* Added new proofs to ` Data.Sum.Properties ` :
482
482
``` agda
483
483
map-id : map id id ≗ id
@@ -616,12 +616,12 @@ Other minor additions
616
616
_on₂_ : (C → C → D) → (A → B → C) → (A → B → D)
617
617
```
618
618
619
- * Added new function in ` Function.Bundles ` :
619
+ * Added new proofs to ` Function.Bundles ` :
620
620
``` agda
621
621
mk↔′ : ∀ (f : A → B) (f⁻¹ : B → A) → Inverseˡ f f⁻¹ → Inverseʳ f f⁻¹ → A ↔ B
622
622
```
623
623
624
- * Added new operator to ` Relation.Binary ` :
624
+ * Added new operators to ` Relation.Binary ` :
625
625
``` agda
626
626
_⇔_ : REL A B ℓ₁ → REL A B ℓ₂ → Set _
627
627
```
@@ -642,7 +642,7 @@ Other minor additions
642
642
icong′ : {f : A → B} x → f x ≡ f x
643
643
```
644
644
645
- * Added new proof to ` Relation.Nullary.Decidable ` :
645
+ * Added new proofs to ` Relation.Nullary.Decidable ` :
646
646
``` agda
647
647
True-↔ : (dec : Dec P) → Irrelevant P → True dec ↔ P
648
648
```
@@ -652,7 +652,7 @@ Other minor additions
652
652
<-isDecStrictPartialOrder : IsDecPartialOrder _≈_ _≤_ → IsDecStrictPartialOrder _≈_ _<_
653
653
```
654
654
655
- * The following operators have had fixities assigneed :
655
+ * The following operators have had fixities assigned :
656
656
```
657
657
infix 4 _[_] (Data.Graph.Acyclic)
658
658
0 commit comments