Skip to content

Commit d85cd7e

Browse files
Minor tidying up of CHANGELOG and prep for v2.2-rc1 (#2540)
* Minor changes to CHANGELOG and prep for v2.2-rc1 * Fix James' comment
1 parent 513117b commit d85cd7e

File tree

3 files changed

+53
-45
lines changed

3 files changed

+53
-45
lines changed

CHANGELOG.md

+46-38
Original file line numberDiff line numberDiff line change
@@ -1,41 +1,41 @@
1-
Version 2.2-dev
2-
===============
1+
Version 2.2
2+
===========
33

4-
The library has been tested using Agda 2.7.0.
4+
The library has been tested using Agda 2.7.0 and 2.7.0.1.
55

66
Highlights
77
----------
88

9+
* Added missing morphisms between the more advanced algebraic structures.
10+
11+
* Added many missing lemmas about positive and negative rational numbers.
12+
913
Bug-fixes
1014
---------
1115

12-
* Relax the types for `≡-syntax` in `Relation.Binary.HeterogeneousEquality`.
16+
* Made the types for `≡-syntax` in `Relation.Binary.HeterogeneousEquality` more general.
1317
These operators are used for equational reasoning of heterogeneous equality
14-
`x ≅ y`, but previously the three operators in `≡-syntax` unnecessarily require
15-
`x` and `y` to have the same type, making them unusable in most situations.
18+
`x ≅ y`, but previously the three operators in `≡-syntax` unnecessarily required
19+
`x` and `y` to have the same type, making them unusable in many situations.
1620

1721
* Removed unnecessary parameter `#-trans : Transitive _#_` from
1822
`Relation.Binary.Reasoning.Base.Apartness`.
1923

24+
* The `IsSemiringWithoutOne` record no longer incorrectly exposes the `Carrier` field
25+
inherited from `Setoid` when opening the record publicly.
26+
2027
Non-backwards compatible changes
2128
--------------------------------
2229

23-
* 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.
24-
25-
* The names exposed by the `IsSemiringWithoutOne` record have been altered to
26-
better correspond to other algebraic structures. In particular:
27-
* `Carrier` is no longer exposed.
28-
* Several laws have been re-exposed from `IsCommutativeMonoid +` renaming
29-
them to name the operation `+`.
30-
* `distribˡ` and `distribʳ` are defined in the record.
30+
* 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 majority of uses, and would only be non-backwards compatible if for some reason you were explicitly supplying these implicit parameters when importing the module. Explicitly supplying the implicit parameters for functions exported from the module should not be affected.
3131

32-
* [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.
33-
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.
32+
* [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. This should be a backwards compatible change for the majority of uses, but the change in parametrisation means that these patterns are *not* necessarily well-formed if the old implicit arguments `m`,`n` are supplied explicitly.
3533

3634
Minor improvements
3735
------------------
3836

37+
* 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.
38+
3939
Deprecated modules
4040
------------------
4141

@@ -111,7 +111,7 @@ New modules
111111
-----------
112112

113113
* Consequences of module monomorphisms
114-
```agda
114+
```
115115
Algebra.Module.Morphism.BimoduleMonomorphism
116116
Algebra.Module.Morphism.BisemimoduleMonomorphism
117117
Algebra.Module.Morphism.LeftModuleMonomorphism
@@ -128,36 +128,28 @@ New modules
128128
```
129129

130130
* Properties of `IdempotentCommutativeMonoid`s refactored out from `Algebra.Solver.IdempotentCommutativeMonoid`:
131-
```agda
131+
```
132132
Algebra.Properties.IdempotentCommutativeMonoid
133133
```
134134

135135
* Refactoring of the `Algebra.Solver.*Monoid` implementations, via
136136
a single `Solver` module API based on the existing `Expr`, and
137137
a common `Normal`-form API:
138-
```agda
138+
```
139139
Algebra.Solver.CommutativeMonoid.Normal
140140
Algebra.Solver.IdempotentCommutativeMonoid.Normal
141141
Algebra.Solver.Monoid.Expression
142142
Algebra.Solver.Monoid.Normal
143143
Algebra.Solver.Monoid.Solver
144144
```
145-
146145
NB Imports of the existing proof procedures `solve` and `prove` etc. should still be via the top-level interfaces in `Algebra.Solver.*Monoid`.
147146

148-
* `Data.List.Effectful.Foldable`: `List` is `Foldable`
149-
150147
* `Data.List.Relation.Binary.Disjoint.Propositional.Properties`:
151148
Propositional counterpart to `Data.List.Relation.Binary.Disjoint.Setoid.Properties`
152-
```agda
153-
sum-↭ : sum Preserves _↭_ ⟶ _≡_
154-
```
155149

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
150+
* Properties of list permutations that require the `--with-K` flag:
151+
```
152+
Data.List.Relation.Binary.Permutation.Propositional.Properties.WithK
161153
```
162154

163155
* Refactored `Data.Refinement` into:
@@ -166,15 +158,17 @@ New modules
166158
Data.Refinement.Properties
167159
```
168160

169-
* `Data.Vec.Effectful.Foldable`: `Vec` is `Foldable`
170-
171-
* `Effect.Foldable`: implementation of haskell-like `Foldable`
161+
* Added implementation of Haskell-like `Foldable`:
162+
```agda
163+
Effect.Foldable
164+
Data.List.Effectful.Foldable
165+
Data.Vec.Effectful.Foldable
166+
```
172167

173168
* Raw bundles for the `Relation.Binary.Bundles` hierarchy:
174169
```agda
175170
Relation.Binary.Bundles.Raw
176171
```
177-
plus adding `rawX` fields to each of `Relation.Binary.Bundles.X`.
178172

179173
Additions to existing modules
180174
-----------------------------
@@ -271,6 +265,19 @@ Additions to existing modules
271265
isNearSemiringHomomorphism : IsNearSemiringHomomorphism ⟦_⟧
272266
```
273267

268+
* In `Algebra.Structures.IsSemiringWithoutOne`:
269+
```agda
270+
distribˡ : * DistributesOverˡ +
271+
distribʳ : * DistributesOverʳ +
272+
+-cong : Congruent +
273+
+-congˡ : LeftCongruent +
274+
+-congʳ : RightCongruent +
275+
+-assoc : Associative +
276+
+-identity : Identity 0# +
277+
+-identityˡ : LeftIdentity 0# +
278+
+-identityʳ : RightIdentity 0# +
279+
```
280+
274281
* Properties of non-divisibility in `Algebra.Properties.Magma.Divisibility`:
275282
```agda
276283
∤-respˡ-≈ : _∤_ Respectsˡ _≈_
@@ -338,9 +345,7 @@ Additions to existing modules
338345
concatMap-++ : concatMap f (xs ++ ys) ≡ concatMap f xs ++ concatMap f ys
339346
filter-≐ : P ≐ Q → filter P? ≗ filter Q?
340347
341-
partition-is-foldr : partition P? ≗ foldr (λ x → if does (P? x) then Product.map₁ (x ∷_)
342-
else Product.map₂ (x ∷_))
343-
([] , [])
348+
partition-is-foldr : partition P? ≗ foldr (λ x → if does (P? x) then map₁ (x ∷_) else map₂ (x ∷_)) ([] , [])
344349
```
345350

346351
* In `Data.List.Relation.Binary.Disjoint.Propositional.Properties`:
@@ -386,6 +391,7 @@ Additions to existing modules
386391
∈-resp-[σ∘σ⁻¹] : (σ : xs ↭ ys) (iy : y ∈ ys) →
387392
∈-resp-↭ (trans (↭-sym σ) σ) iy ≡ iy
388393
product-↭ : product Preserves _↭_ ⟶ _≡_
394+
sum-↭ : sum Preserves _↭_ ⟶ _≡_
389395
```
390396

391397
* In `Data.List.Relation.Binary.Permutation.Propositional.Properties.WithK`:
@@ -595,6 +601,8 @@ Additions to existing modules
595601
```
596602
plus associated `isDecPreorder` fields in each higher `IsDec*Order` structure.
597603

604+
* In `Relation.Binary.Bundles` added `rawX` (e.g. `RawSetoid`) fields to each bundle.
605+
598606
* In `Relation.Nullary.Decidable`:
599607
```agda
600608
does-⇔ : A ⇔ B → (a? : Dec A) → (b? : Dec B) → does a? ≡ does b?

LICENCE

+1-1
Original file line numberDiff line numberDiff line change
@@ -1,4 +1,4 @@
1-
Copyright (c) 2007-2024 Nils Anders Danielsson, Ulf Norell, Shin-Cheng
1+
Copyright (c) 2007-2025 Nils Anders Danielsson, Ulf Norell, Shin-Cheng
22
Mu, Bradley Hardy, Samuel Bronson, Dan Doel, Patrik Jansson,
33
Liang-Ting Chen, Jean-Philippe Bernardy, Andrés Sicard-Ramírez,
44
Nicolas Pouillard, Darin Morrison, Peter Berry, Daniel Brown,

doc/installation-guide.md

+6-6
Original file line numberDiff line numberDiff line change
@@ -3,19 +3,19 @@ Installation instructions
33

44
Note: the full story on installing Agda libraries can be found at [readthedocs](http://agda.readthedocs.io/en/latest/tools/package-system.html).
55

6-
Use version v2.1.1 of the standard library with Agda 2.7.0. You can find the correct version of the library to use for different Agda versions on the [Agda Wiki](https://wiki.portal.chalmers.se/agda/Libraries/StandardLibrary).
6+
Use version v2.2 of the standard library with Agda v2.7.0 or v2.7.0.1. You can find the correct version of the library to use for different Agda versions on the [Agda Wiki](https://wiki.portal.chalmers.se/agda/Libraries/StandardLibrary).
77

88
1. Navigate to a suitable directory `$HERE` (replace appropriately) where
99
you would like to install the library.
1010

11-
2. Download the tarball of v2.1.1 of the standard library. This can either be
11+
2. Download the tarball of v2.2 of the standard library. This can either be
1212
done manually by visiting the Github repository for the library, or via the
1313
command line as follows:
1414
```
15-
wget -O agda-stdlib.tar.gz https://github.com/agda/agda-stdlib/archive/v2.1.1.tar.gz
15+
wget -O agda-stdlib.tar.gz https://github.com/agda/agda-stdlib/archive/v2.2.tar.gz
1616
```
1717
Note that you can replace `wget` with other popular tools such as `curl` and that
18-
you can replace `2.1.1` with any other version of the library you desire.
18+
you can replace `2.2` with any other version of the library you desire.
1919

2020
3. Extract the standard library from the tarball. Again this can either be
2121
done manually or via the command line as follows:
@@ -26,7 +26,7 @@ Use version v2.1.1 of the standard library with Agda 2.7.0. You can find the cor
2626
4. [ OPTIONAL ] If using [cabal](https://www.haskell.org/cabal/) then run
2727
the commands to install via cabal:
2828
```
29-
cd agda-stdlib-2.1.1
29+
cd agda-stdlib-2.2
3030
cabal install
3131
```
3232

@@ -42,7 +42,7 @@ Use version v2.1.1 of the standard library with Agda 2.7.0. You can find the cor
4242
6. Register the standard library with Agda's package system by adding
4343
the following line to `$AGDA_DIR/libraries`:
4444
```
45-
$HERE/agda-stdlib-2.1.1/standard-library.agda-lib
45+
$HERE/agda-stdlib-2.2/standard-library.agda-lib
4646
```
4747

4848
Now, the standard library is ready to be used either:

0 commit comments

Comments
 (0)