You signed in with another tab or window. Reload to refresh your session.You signed out in another tab or window. Reload to refresh your session.You switched accounts on another tab or window. Reload to refresh your session.Dismiss alert
Copy file name to clipboardExpand all lines: CHANGELOG.md
+46-38
Original file line number
Diff line number
Diff line change
@@ -1,41 +1,41 @@
1
-
Version 2.2-dev
2
-
===============
1
+
Version 2.2
2
+
===========
3
3
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.
5
5
6
6
Highlights
7
7
----------
8
8
9
+
* Added missing morphisms between the more advanced algebraic structures.
10
+
11
+
* Added many missing lemmas about positive and negative rational numbers.
12
+
9
13
Bug-fixes
10
14
---------
11
15
12
-
*Relax the types for `≡-syntax` in `Relation.Binary.HeterogeneousEquality`.
16
+
*Made the types for `≡-syntax` in `Relation.Binary.HeterogeneousEquality` more general.
13
17
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.
16
20
17
21
* Removed unnecessary parameter `#-trans : Transitive _#_` from
18
22
`Relation.Binary.Reasoning.Base.Apartness`.
19
23
24
+
* The `IsSemiringWithoutOne` record no longer incorrectly exposes the `Carrier` field
25
+
inherited from `Setoid` when opening the record publicly.
26
+
20
27
Non-backwards compatible changes
21
28
--------------------------------
22
29
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.
31
31
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.
35
33
36
34
Minor improvements
37
35
------------------
38
36
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
+
39
39
Deprecated modules
40
40
------------------
41
41
@@ -111,7 +111,7 @@ New modules
111
111
-----------
112
112
113
113
* Consequences of module monomorphisms
114
-
```agda
114
+
```
115
115
Algebra.Module.Morphism.BimoduleMonomorphism
116
116
Algebra.Module.Morphism.BisemimoduleMonomorphism
117
117
Algebra.Module.Morphism.LeftModuleMonomorphism
@@ -128,36 +128,28 @@ New modules
128
128
```
129
129
130
130
* Properties of `IdempotentCommutativeMonoid`s refactored out from `Algebra.Solver.IdempotentCommutativeMonoid`:
131
-
```agda
131
+
```
132
132
Algebra.Properties.IdempotentCommutativeMonoid
133
133
```
134
134
135
135
* Refactoring of the `Algebra.Solver.*Monoid` implementations, via
136
136
a single `Solver` module API based on the existing `Expr`, and
137
137
a common `Normal`-form API:
138
-
```agda
138
+
```
139
139
Algebra.Solver.CommutativeMonoid.Normal
140
140
Algebra.Solver.IdempotentCommutativeMonoid.Normal
141
141
Algebra.Solver.Monoid.Expression
142
142
Algebra.Solver.Monoid.Normal
143
143
Algebra.Solver.Monoid.Solver
144
144
```
145
-
146
145
NB Imports of the existing proof procedures `solve` and `prove` etc. should still be via the top-level interfaces in `Algebra.Solver.*Monoid`.
147
146
148
-
*`Data.List.Effectful.Foldable`: `List` is `Foldable`
Copy file name to clipboardExpand all lines: doc/installation-guide.md
+6-6
Original file line number
Diff line number
Diff line change
@@ -3,19 +3,19 @@ Installation instructions
3
3
4
4
Note: the full story on installing Agda libraries can be found at [readthedocs](http://agda.readthedocs.io/en/latest/tools/package-system.html).
5
5
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).
7
7
8
8
1. Navigate to a suitable directory `$HERE` (replace appropriately) where
9
9
you would like to install the library.
10
10
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
12
12
done manually by visiting the Github repository for the library, or via the
0 commit comments