Skip to content

Commit 11d0a33

Browse files
authored
[ fix ] tidy up alphabetical ordering in CHANGELOG (agda#2538)
* tidy up alphabetical ordering * refactor: more comprehensive overhaul
1 parent d481f5c commit 11d0a33

File tree

1 file changed

+87
-92
lines changed

1 file changed

+87
-92
lines changed

CHANGELOG.md

Lines changed: 87 additions & 92 deletions
Original file line numberDiff line numberDiff line change
@@ -9,18 +9,17 @@ Highlights
99
Bug-fixes
1010
---------
1111

12-
* Removed unnecessary parameter `#-trans : Transitive _#_` from
13-
`Relation.Binary.Reasoning.Base.Apartness`.
1412
* Relax the types for `≡-syntax` in `Relation.Binary.HeterogeneousEquality`.
1513
These operators are used for equational reasoning of heterogeneous equality
1614
`x ≅ y`, but previously the three operators in `≡-syntax` unnecessarily require
1715
`x` and `y` to have the same type, making them unusable in most situations.
1816

17+
* Removed unnecessary parameter `#-trans : Transitive _#_` from
18+
`Relation.Binary.Reasoning.Base.Apartness`.
19+
1920
Non-backwards compatible changes
2021
--------------------------------
2122

22-
* In `Function.Related.TypeIsomorphisms`, the unprimed versions are more level polymorphic; and the primed versions retain `Level` homogeneous types for the `Semiring` axioms to hold.
23-
2423
* In `Data.List.Relation.Binary.Sublist.Propositional.Properties` the implicit module parameters `a` and `A` have been replaced with `variable`s. This should be a backwards compatible change for the overwhelming majority of uses, and would only be non-backwards compatible if you were explicitly supplying these implicit parameters for some reason when importing the module. Explicitly supplying the implicit parameters for functions exported from the module should not be affected.
2524

2625
* The names exposed by the `IsSemiringWithoutOne` record have been altered to
@@ -32,6 +31,8 @@ Non-backwards compatible changes
3231

3332
* [issue #2504](https://github.com/agda/agda-stdlib/issues/2504) and [issue #2519](https://github.com/agda/agda-stdlib/issues/2510) In `Data.Nat.Base` the definitions of `_≤′_` and `_≤‴_` have been modified to make the witness to equality explicit in new constructors `≤′-reflexive` and `≤‴-reflexive`; pattern synonyms `≤′-refl` and `≤‴-refl` have been added for backwards compatibility but NB. the change in parametrisation means that these patterns are *not* necessarily well-formed if the old implicit arguments `m`,`n` are supplied explicitly.
3433

34+
* In `Function.Related.TypeIsomorphisms`, the unprimed versions are more level polymorphic; and the primed versions retain `Level` homogeneous types for the `Semiring` axioms to hold.
35+
3536
Minor improvements
3637
------------------
3738

@@ -109,16 +110,6 @@ Deprecated names
109110
New modules
110111
-----------
111112

112-
* Bundled morphisms between (raw) algebraic structures:
113-
```
114-
Algebra.Morphism.Bundles
115-
```
116-
117-
* Properties of `IdempotentCommutativeMonoid`s refactored out from `Algebra.Solver.IdempotentCommutativeMonoid`:
118-
```agda
119-
Algebra.Properties.IdempotentCommutativeMonoid
120-
```
121-
122113
* Consequences of module monomorphisms
123114
```agda
124115
Algebra.Module.Morphism.BimoduleMonomorphism
@@ -131,6 +122,16 @@ New modules
131122
Algebra.Module.Morphism.SemimoduleMonomorphism
132123
```
133124

125+
* Bundled morphisms between (raw) algebraic structures:
126+
```
127+
Algebra.Morphism.Bundles
128+
```
129+
130+
* Properties of `IdempotentCommutativeMonoid`s refactored out from `Algebra.Solver.IdempotentCommutativeMonoid`:
131+
```agda
132+
Algebra.Properties.IdempotentCommutativeMonoid
133+
```
134+
134135
* Refactoring of the `Algebra.Solver.*Monoid` implementations, via
135136
a single `Solver` module API based on the existing `Expr`, and
136137
a common `Normal`-form API:
@@ -144,37 +145,37 @@ New modules
144145

145146
NB Imports of the existing proof procedures `solve` and `prove` etc. should still be via the top-level interfaces in `Algebra.Solver.*Monoid`.
146147

147-
* Refactored out from `Data.List.Relation.Unary.All.Properties` in order to break a dependency cycle with `Data.List.Membership.Setoid.Properties`:
148-
```agda
149-
Data.List.Relation.Unary.All.Properties.Core
150-
```
148+
* `Data.List.Effectful.Foldable`: `List` is `Foldable`
151149

152150
* `Data.List.Relation.Binary.Disjoint.Propositional.Properties`:
153151
Propositional counterpart to `Data.List.Relation.Binary.Disjoint.Setoid.Properties`
154152
```agda
155153
sum-↭ : sum Preserves _↭_ ⟶ _≡_
156154
```
157155

158-
* `Data.List.Relation.Binary.Permutation.Propositional.Properties.WithK`
156+
* Added `Data.List.Relation.Binary.Permutation.Propositional.Properties.WithK`
157+
158+
* Refactored out from `Data.List.Relation.Unary.All.Properties` in order to break a dependency cycle with `Data.List.Membership.Setoid.Properties`:
159+
```agda
160+
Data.List.Relation.Unary.All.Properties.Core
161+
```
159162

160163
* Refactored `Data.Refinement` into:
161164
```agda
162165
Data.Refinement.Base
163166
Data.Refinement.Properties
164167
```
165168

169+
* `Data.Vec.Effectful.Foldable`: `Vec` is `Foldable`
170+
171+
* `Effect.Foldable`: implementation of haskell-like `Foldable`
172+
166173
* Raw bundles for the `Relation.Binary.Bundles` hierarchy:
167174
```agda
168175
Relation.Binary.Bundles.Raw
169176
```
170177
plus adding `rawX` fields to each of `Relation.Binary.Bundles.X`.
171178

172-
* `Data.List.Effectful.Foldable`: `List` is `Foldable`
173-
174-
* `Data.Vec.Effectful.Foldable`: `Vec` is `Foldable`
175-
176-
* `Effect.Foldable`: implementation of haskell-like `Foldable`
177-
178179
Additions to existing modules
179180
-----------------------------
180181

@@ -292,22 +293,6 @@ Additions to existing modules
292293
isNearSemiring : IsNearSemiring _ _
293294
```
294295

295-
* In `Data.List.Membership.Setoid.Properties`:
296-
```agda
297-
∉⇒All[≉] : x ∉ xs → All (x ≉_) xs
298-
All[≉]⇒∉ : All (x ≉_) xs → x ∉ xs
299-
Any-∈-swap : Any (_∈ ys) xs → Any (_∈ xs) ys
300-
All-∉-swap : All (_∉ ys) xs → All (_∉ xs) ys
301-
∈-map∘filter⁻ : y ∈₂ map f (filter P? xs) → ∃[ x ] x ∈₁ xs × y ≈₂ f x × P x
302-
∈-map∘filter⁺ : f Preserves _≈₁_ ⟶ _≈₂_ →
303-
∃[ x ] x ∈₁ xs × y ≈₂ f x × P x →
304-
y ∈₂ map f (filter P? xs)
305-
∈-concatMap⁺ : Any ((y ∈_) ∘ f) xs → y ∈ concatMap f xs
306-
∈-concatMap⁻ : y ∈ concatMap f xs → Any ((y ∈_) ∘ f) xs
307-
∉[] : x ∉ []
308-
deduplicate-∈⇔ : _≈_ Respectsʳ (flip R) → z ∈ xs ⇔ z ∈ deduplicate R? xs
309-
```
310-
311296
* In `Data.List.Membership.Propositional.Properties`:
312297
```agda
313298
∈-AllPairs₂ : AllPairs R xs → x ∈ xs → y ∈ xs → x ≡ y ⊎ R x y ⊎ R y x
@@ -329,6 +314,22 @@ Additions to existing modules
329314
unique∧set⇒bag : Unique xs → Unique ys → xs ∼[ set ] ys → xs ∼[ bag ] ys
330315
```
331316

317+
* In `Data.List.Membership.Setoid.Properties`:
318+
```agda
319+
∉⇒All[≉] : x ∉ xs → All (x ≉_) xs
320+
All[≉]⇒∉ : All (x ≉_) xs → x ∉ xs
321+
Any-∈-swap : Any (_∈ ys) xs → Any (_∈ xs) ys
322+
All-∉-swap : All (_∉ ys) xs → All (_∉ xs) ys
323+
∈-map∘filter⁻ : y ∈₂ map f (filter P? xs) → ∃[ x ] x ∈₁ xs × y ≈₂ f x × P x
324+
∈-map∘filter⁺ : f Preserves _≈₁_ ⟶ _≈₂_ →
325+
∃[ x ] x ∈₁ xs × y ≈₂ f x × P x →
326+
y ∈₂ map f (filter P? xs)
327+
∈-concatMap⁺ : Any ((y ∈_) ∘ f) xs → y ∈ concatMap f xs
328+
∈-concatMap⁻ : y ∈ concatMap f xs → Any ((y ∈_) ∘ f) xs
329+
∉[] : x ∉ []
330+
deduplicate-∈⇔ : _≈_ Respectsʳ (flip R) → z ∈ xs ⇔ z ∈ deduplicate R? xs
331+
```
332+
332333
* In `Data.List.Properties`:
333334
```agda
334335
product≢0 : All NonZero ns → NonZero (product ns)
@@ -342,37 +343,14 @@ Additions to existing modules
342343
([] , [])
343344
```
344345

345-
* In `Data.List.Relation.Binary.Sublist.Propositional.Properties`:
346-
```agda
347-
⊆⇒⊆ₛ : (S : Setoid a ℓ) → as ⊆ bs → as (SetoidSublist.⊆ S) bs
348-
```
349-
350-
* In `Data.List.Relation.Binary.Sublist.Setoid.Properties`:
351-
```agda
352-
concat⁺ : Sublist _⊆_ ass bss → concat ass ⊆ concat bss
353-
all⊆concat : (xss : List (List A)) → All (Sublist._⊆ concat xss) xss
354-
```
355-
356-
* In `Data.List.Relation.Unary.All.Properties`:
357-
```agda
358-
all⇒dropWhile≡[] : (P? : Decidable P) → All P xs → dropWhile P? xs ≡ []
359-
all⇒takeWhile≗id : (P? : Decidable P) → All P xs → takeWhile P? xs ≡ xs
360-
```
361-
362-
* In `Data.List.Relation.Unary.Any.Properties`:
363-
```agda
364-
concatMap⁺ : Any (Any P ∘ f) xs → Any P (concatMap f xs)
365-
concatMap⁻ : Any P (concatMap f xs) → Any (Any P ∘ f) xs
366-
```
367-
368-
* In `Data.List.Relation.Unary.Unique.Setoid.Properties`:
346+
* In `Data.List.Relation.Binary.Disjoint.Propositional.Properties`:
369347
```agda
370-
Unique[x∷xs]⇒x∉xs : Unique S (x ∷ xs) → x ∉ xs
348+
deduplicate⁺ : Disjoint xs ys → Disjoint (deduplicate _≟_ xs) (deduplicate _≟_ ys)
371349
```
372350

373-
* In `Data.List.Relation.Unary.Unique.Propositional.Properties`:
351+
* In `Data.List.Relation.Binary.Disjoint.Setoid.Properties`:
374352
```agda
375-
Unique[x∷xs]⇒x∉xs : Unique (x ∷ xs) → x ∉ xs
353+
deduplicate⁺ : Disjoint S xs ys → Disjoint S (deduplicate _≟_ xs) (deduplicate _≟_ ys)
376354
```
377355

378356
* In `Data.List.Relation.Binary.Equality.Setoid`:
@@ -410,6 +388,12 @@ Additions to existing modules
410388
product-↭ : product Preserves _↭_ ⟶ _≡_
411389
```
412390

391+
* In `Data.List.Relation.Binary.Permutation.Propositional.Properties.WithK`:
392+
```agda
393+
dedup-++-↭ : Disjoint xs ys →
394+
deduplicate _≟_ (xs ++ ys) ↭ deduplicate _≟_ xs ++ deduplicate _≟_ ys
395+
```
396+
413397
* In `Data.List.Relation.Binary.Permutation.Setoid`:
414398
```agda
415399
↭-reflexive-≋ : _≋_ ⇒ _↭_
@@ -431,60 +415,71 @@ Additions to existing modules
431415
++⁺ʳ : Reflexive R → ∀ zs → (_++ zs) Preserves (Pointwise R) ⟶ (Pointwise R)
432416
```
433417

434-
* In `Data.List.Relation.Unary.All`:
418+
* In `Data.List.Relation.Binary.Sublist.Heterogeneous.Properties`:
435419
```agda
436-
search : Decidable P → ∀ xs → All (∁ P) xs ⊎ Any P xs
437-
```
420+
Sublist-[]-universal : Universal (Sublist R [])
421+
```
438422

439-
* In `Data.List.Relation.Binary.Subset.Setoid.Properties`:
423+
* In `Data.List.Relation.Binary.Sublist.Propositional.Properties`:
440424
```agda
441-
∷⊈[] : x ∷ xs ⊈ []
442-
⊆∷⇒∈∨⊆ : xs ⊆ y ∷ ys → y ∈ xs ⊎ xs ⊆ ys
443-
⊆∷∧∉⇒⊆ : xs ⊆ y ∷ ys → y ∉ xs → xs ⊆ ys
425+
⊆⇒⊆ₛ : (S : Setoid a ℓ) → as ⊆ bs → as (SetoidSublist.⊆ S) bs
426+
```
427+
428+
* In `Data.List.Relation.Binary.Sublist.Setoid.Properties`:
429+
```agda
430+
[]⊆-universal : Universal ([] ⊆_)
431+
432+
concat⁺ : Sublist _⊆_ ass bss → concat ass ⊆ concat bss
433+
all⊆concat : (xss : List (List A)) → All (Sublist._⊆ concat xss) xss
444434
```
445435

446436
* In `Data.List.Relation.Binary.Subset.Propositional.Properties`:
447437
```agda
448438
∷⊈[] : x ∷ xs ⊈ []
449439
⊆∷⇒∈∨⊆ : xs ⊆ y ∷ ys → y ∈ xs ⊎ xs ⊆ ys
450440
⊆∷∧∉⇒⊆ : xs ⊆ y ∷ ys → y ∉ xs → xs ⊆ ys
441+
442+
concatMap⁺ : xs ⊆ ys → concatMap f xs ⊆ concatMap f ys
451443
```
452444

453-
* In `Data.List.Relation.Binary.Subset.Propositional.Properties`:
445+
* In `Data.List.Relation.Binary.Subset.Setoid.Properties`:
454446
```agda
455-
concatMap⁺ : xs ⊆ ys → concatMap f xs ⊆ concatMap f ys
447+
∷⊈[] : x ∷ xs ⊈ []
448+
⊆∷⇒∈∨⊆ : xs ⊆ y ∷ ys → y ∈ xs ⊎ xs ⊆ ys
449+
⊆∷∧∉⇒⊆ : xs ⊆ y ∷ ys → y ∉ xs → xs ⊆ ys
456450
```
457451

458-
* In `Data.List.Relation.Binary.Sublist.Heterogeneous.Properties`:
452+
* In `Data.List.Relation.Unary.First.Properties`:
459453
```agda
460-
Sublist-[]-universal : Universal (Sublist R [])
454+
¬First⇒All : ∁ Q ⊆ P → ∁ (First P Q) ⊆ All P
455+
¬All⇒First : Decidable P → ∁ P ⊆ Q → ∁ (All P) ⊆ First P Q
461456
```
462457

463-
* In `Data.List.Relation.Binary.Sublist.Setoid.Properties`:
458+
* In `Data.List.Relation.Unary.All`:
464459
```agda
465-
[]⊆-universal : Universal ([] ⊆_)
460+
search : Decidable P → ∀ xs → All (∁ P) xs ⊎ Any P xs
466461
```
467462

468-
* In `Data.List.Relation.Binary.Disjoint.Setoid.Properties`:
463+
* In `Data.List.Relation.Unary.All.Properties`:
469464
```agda
470-
deduplicate⁺ : Disjoint S xs ys → Disjoint S (deduplicate _≟_ xs) (deduplicate _≟_ ys)
465+
all⇒dropWhile≡[] : (P? : Decidable P) → All P xs → dropWhile P? xs ≡ []
466+
all⇒takeWhile≗id : (P? : Decidable P) → All P xs → takeWhile P? xs ≡ xs
471467
```
472468

473-
* In `Data.List.Relation.Binary.Disjoint.Propositional.Properties`:
469+
* In `Data.List.Relation.Unary.Any.Properties`:
474470
```agda
475-
deduplicate⁺ : Disjoint xs ys → Disjoint (deduplicate _≟_ xs) (deduplicate _≟_ ys)
471+
concatMap⁺ : Any (Any P ∘ f) xs → Any P (concatMap f xs)
472+
concatMap⁻ : Any P (concatMap f xs) → Any (Any P ∘ f) xs
476473
```
477474

478-
* In `Data.List.Relation.Binary.Permutation.Propositional.Properties.WithK`:
475+
* In `Data.List.Relation.Unary.Unique.Propositional.Properties`:
479476
```agda
480-
dedup-++-↭ : Disjoint xs ys →
481-
deduplicate _≟_ (xs ++ ys) ↭ deduplicate _≟_ xs ++ deduplicate _≟_ ys
477+
Unique[x∷xs]⇒x∉xs : Unique (x ∷ xs) → x ∉ xs
482478
```
483479

484-
* In `Data.List.Relation.Unary.First.Properties`:
480+
* In `Data.List.Relation.Unary.Unique.Setoid.Properties`:
485481
```agda
486-
¬First⇒All : ∁ Q ⊆ P → ∁ (First P Q) ⊆ All P
487-
¬All⇒First : Decidable P → ∁ P ⊆ Q → ∁ (All P) ⊆ First P Q
482+
Unique[x∷xs]⇒x∉xs : Unique S (x ∷ xs) → x ∉ xs
488483
```
489484

490485
* In `Data.Maybe.Properties`:
@@ -503,7 +498,7 @@ Additions to existing modules
503498
≥‴-irrelevant : Irrelevant {A = ℕ} _≥‴_
504499
```
505500

506-
adjunction between `suc` and `pred`
501+
Added adjunction between `suc` and `pred`
507502
```agda
508503
suc[m]≤n⇒m≤pred[n] : suc m ≤ n → m ≤ pred n
509504
m≤pred[n]⇒suc[m]≤n : .{{NonZero n}} → m ≤ pred n → suc m ≤ n

0 commit comments

Comments
 (0)