Skip to content

Commit 0a7119c

Browse files
Updated CHANGELOG for final changes for v1.4
1 parent 8483681 commit 0a7119c

File tree

3 files changed

+64
-64
lines changed

3 files changed

+64
-64
lines changed

CHANGELOG.md

+54-54
Original file line numberDiff line numberDiff line change
@@ -21,24 +21,23 @@ Bug-fixes
2121
* Fixed various algebraic bundles not correctly re-exporting
2222
`commutativeSemigroup` proofs.
2323

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
2525
the predicate `P` were required to live at the same universe level.
2626

2727
Non-backwards compatible changes
2828
--------------------------------
2929

3030
#### Changes to the `Relation.Unary.Closure` hierarchy
3131

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
3435

3536
+ 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`)
4139

40+
* Added functions converting back and forth between ``-based and ``-based statements in `.Base`:
4241
```agda
4342
curry : (∀ {x} → ◇ T x → P x) → (∀ {x} → T x → □ P x)
4443
uncurry : (∀ {x} → T x → □ P x) → (∀ {x} → ◇ T x → P x)
@@ -48,31 +47,34 @@ Non-backwards compatible changes
4847

4948
* The `n` argument to `_⊜_` in `Tactic.RingSolver.NonReflective` has been made implict rather than explicit.
5049

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.
5656

5757
Deprecated modules
5858
------------------
5959

60-
* `Data.AVL` and all of its submodules have been moved to `Data.Tree.AVL`
61-
6260
* The module `Induction.WellFounded.InverseImage` has been deprecated. The proofs
6361
`accessible` and `wellFounded` have been moved to `Relation.Binary.Construct.On`.
6462

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`.
6667

6768
Deprecated names
6869
----------------
6970

7071
* The proofs `replace-equality` from `Algebra.Properties.(Lattice/DistributiveLattice/BooleanAlgebra)`
7172
have been deprecated in favour of the proofs in the new `Algebra.Construct.Subst.Equality` module.
7273

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._∷ʳ′_`
7678
* `Relation.Binary.Construct.StrictToNonStrict.decidable'``Relation.Binary.Construct.StrictToNonStrict.decidable′`
7779

7880
* In `Algebra.Morphism.Definitions` and `Relation.Binary.Morphism.Definitions`
@@ -95,15 +97,19 @@ Deprecated names
9597
*-+-commutativeSemiring ↦ +-*-commutativeSemiring
9698
*-+-isSemiringWithoutAnnihilatingZero ↦ +-*-isSemiringWithoutAnnihilatingZero
9799
```
98-
* In ̀Function.Basè:
100+
101+
* In `Function.Base`:
99102
```
100103
*_-[_]-_ ↦ _-⟪_⟫-_
101104
```
102105

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?`
107113

108114
New modules
109115
-----------
@@ -115,7 +121,7 @@ New modules
115121
Algebra.Module.Construct.DirectProduct.agda
116122
```
117123

118-
* Substituting the notion of equality for various structures
124+
* Substituting the notion of equality for various structures:
119125
```
120126
Algebra.Construct.Subst.Equality
121127
Relation.Binary.Construct.Subst.Equality
@@ -133,7 +139,7 @@ New modules
133139
Function.Identity.Instances
134140
```
135141

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:
137143
```
138144
Data.List.Relation.Unary.Sorted.TotalOrder
139145
Data.List.Relation.Unary.Sorted.TotalOrder.Properties
@@ -144,13 +150,13 @@ New modules
144150
Data.Nat.Binary.Subtraction
145151
```
146152

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:
148154
```
149155
Data.Vec.Relation.Unary.AllPairs
150156
Data.Vec.Relation.Unary.AllPairs.Properties
151157
```
152158

153-
* A predicate for vectors in which every element is unique.
159+
* A predicate for vectors in which every element is unique:
154160
```
155161
Data.Vec.Relation.Unary.Unique.Propositional
156162
Data.Vec.Relation.Unary.Unique.Propositional.Properties
@@ -171,7 +177,7 @@ New modules
171177
```
172178

173179
* Modules replacing `Function.Related.TypeIsomorphisms` using the new
174-
`Inverse` definitions.
180+
`Inverse` definitions:
175181
```
176182
Data.Sum.Algebra
177183
Data.Product.Algebra
@@ -182,12 +188,12 @@ New modules
182188
Function.Properties
183189
```
184190

185-
* Symmetry for various functional properties
191+
* Symmetry for various functional properties:
186192
```agda
187193
Function.Construct.Symmetry
188194
```
189195

190-
* Added a hierarchy for metric spaces:
196+
* A hierarchy for metric spaces:
191197
```
192198
Function.Metric
193199
Function.Metric.Core
@@ -206,7 +212,7 @@ New modules
206212
```
207213
and other specialisations can be created in a similar fashion.
208214

209-
* Type-checking monads
215+
* The type-checking monads:
210216
```
211217
Reflection.TypeChecking.Monad
212218
Reflection.TypeChecking.Monad.Categorical
@@ -230,7 +236,7 @@ New modules
230236
Relation.Binary.Construct.Composition
231237
```
232238

233-
* Generic printf
239+
* Generic `printf` method:
234240
```
235241
Text.Format.Generic
236242
Text.Printf.Generic
@@ -239,25 +245,24 @@ New modules
239245
Other major changes
240246
-------------------
241247

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:
246253
```agda
247254
Relation.Binary.PropositionalEquality.Properties
248255
Relation.Binary.PropositionalEquality.Algebra
249256
```
250257
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.
253259

254260
Other minor additions
255261
---------------------
256262

257263
* Add proof to `Algebra.Morphism.RingMonomorphism`:
258264
```agda
259-
isCommutativeRing : IsCommutativeRing _≈₂_ _⊕_ _⊛_ ⊝_ 0#₂ 1#₂ →
260-
IsCommutativeRing _≈₁_ _+_ _*_ -_ 0# 1#
265+
isCommutativeRing : IsCommutativeRing _≈₂_ _⊕_ _⊛_ ⊝_ 0#₂ 1#₂ → IsCommutativeRing _≈₁_ _+_ _*_ -_ 0# 1#
261266
```
262267

263268
* Added new proof to `Data.Fin.Induction`:
@@ -269,7 +274,7 @@ Other minor additions
269274
```agda
270275
toℕ≤n : (i : Fin n) → toℕ i ≤ n
271276
≤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
273278
fromℕ<-injective : fromℕ< m<o ≡ fromℕ< n<o → m ≡ n
274279
inject₁ℕ< : (i : Fin n) → toℕ (inject₁ i) < n
275280
inject₁ℕ≤ : (i : Fin n) → toℕ (inject₁ i) ≤ n
@@ -455,12 +460,9 @@ Other minor additions
455460
assocʳ′ : (A × B) × C → A × (B × C)
456461
assocˡ′ : A × (B × C) → (A × B) × C
457462
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
464466
```
465467

466468
* Added new proofs to `Data.Product.Properties`:
@@ -476,8 +478,6 @@ Other minor additions
476478
assocˡ : A ⊎ B ⊎ C → (A ⊎ B) ⊎ C
477479
```
478480

479-
* Made first argument of `[,]-∘-distr` in `Data.Sum.Properties` explicit
480-
481481
* Added new proofs to `Data.Sum.Properties`:
482482
```agda
483483
map-id : map id id ≗ id
@@ -616,12 +616,12 @@ Other minor additions
616616
_on₂_ : (C → C → D) → (A → B → C) → (A → B → D)
617617
```
618618

619-
* Added new function in `Function.Bundles`:
619+
* Added new proofs to `Function.Bundles`:
620620
```agda
621621
mk↔′ : ∀ (f : A → B) (f⁻¹ : B → A) → Inverseˡ f f⁻¹ → Inverseʳ f f⁻¹ → A ↔ B
622622
```
623623

624-
* Added new operator to `Relation.Binary`:
624+
* Added new operators to `Relation.Binary`:
625625
```agda
626626
_⇔_ : REL A B ℓ₁ → REL A B ℓ₂ → Set _
627627
```
@@ -642,7 +642,7 @@ Other minor additions
642642
icong′ : {f : A → B} x → f x ≡ f x
643643
```
644644

645-
* Added new proof to `Relation.Nullary.Decidable`:
645+
* Added new proofs to `Relation.Nullary.Decidable`:
646646
```agda
647647
True-↔ : (dec : Dec P) → Irrelevant P → True dec ↔ P
648648
```
@@ -652,7 +652,7 @@ Other minor additions
652652
<-isDecStrictPartialOrder : IsDecPartialOrder _≈_ _≤_ → IsDecStrictPartialOrder _≈_ _<_
653653
```
654654

655-
* The following operators have had fixities assigneed:
655+
* The following operators have had fixities assigned:
656656
```
657657
infix 4 _[_] (Data.Graph.Acyclic)
658658

src/Data/Fin/Properties.agda

+7-7
Original file line numberDiff line numberDiff line change
@@ -151,13 +151,13 @@ fromℕ-def : ∀ n → fromℕ n ≡ fromℕ< ℕₚ.≤-refl
151151
fromℕ-def zero = refl
152152
fromℕ-def (suc n) = cong suc (fromℕ-def n)
153153

154-
fromℕ<-irrelevant : m n {o} m ≡ n
155-
(m<o : m ℕ.< o)
156-
(n<o : n ℕ.< o)
157-
fromℕ< m<o ≡ fromℕ< n<o
158-
fromℕ<-irrelevant 0 0 r (s≤s z≤n) (s≤s z≤n) = refl
159-
fromℕ<-irrelevant (suc _) (suc _) r (s≤s (s≤s p)) (s≤s (s≤s q))
160-
= cong suc (fromℕ<-irrelevant _ _ (ℕₚ.suc-injective r) (s≤s p) (s≤s q))
154+
fromℕ<-cong : m n {o} m ≡ n
155+
(m<o : m ℕ.< o)
156+
(n<o : n ℕ.< o)
157+
fromℕ< m<o ≡ fromℕ< n<o
158+
fromℕ<-cong 0 0 r (s≤s z≤n) (s≤s z≤n) = refl
159+
fromℕ<-cong (suc _) (suc _) r (s≤s (s≤s p)) (s≤s (s≤s q))
160+
= cong suc (fromℕ<-cong _ _ (ℕₚ.suc-injective r) (s≤s p) (s≤s q))
161161

162162
fromℕ<-injective : m n {o}
163163
(m<o : m ℕ.< o)

src/Data/Product.agda

+3-3
Original file line numberDiff line numberDiff line change
@@ -116,8 +116,8 @@ map₂ f = map id f
116116

117117
-- A version of map where the output can depend on the input
118118
dmap : {B : A Set b} {P : A Set p} {Q : {a} P a B a Set q}
119-
(f : (a : A) B a) ( {a} (p : P a) Q p (f a))
120-
(ap : Σ A P) Σ (B (proj₁ ap)) (Q (proj₂ ap))
119+
(f : (a : A) B a) ( {a} (b : P a) Q b (f a))
120+
((a , b) : Σ A P) Σ (B a) (Q b)
121121
dmap f g (x , y) = f x , g y
122122

123123
zip : {P : A Set p} {Q : B Set q} {R : C Set r}
@@ -175,7 +175,7 @@ uncurry′ = uncurry
175175

176176
dmap′ : {x y} {X : A Set x} {Y : B Set y}
177177
((a : A) X a) ((b : B) Y b)
178-
(ab : A × B) X (proj₁ ab) × Y (proj₂ ab)
178+
((a , b) : A × B) X a × Y b
179179
dmap′ f g = dmap f g
180180

181181
_<*>_ : {x y} {X : A Set x} {Y : B Set y}

0 commit comments

Comments
 (0)