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
+87-92Lines changed: 87 additions & 92 deletions
Display the source diff
Display the rich diff
Original file line number
Diff line number
Diff line change
@@ -9,18 +9,17 @@ Highlights
9
9
Bug-fixes
10
10
---------
11
11
12
-
* Removed unnecessary parameter `#-trans : Transitive _#_` from
13
-
`Relation.Binary.Reasoning.Base.Apartness`.
14
12
* Relax the types for `≡-syntax` in `Relation.Binary.HeterogeneousEquality`.
15
13
These operators are used for equational reasoning of heterogeneous equality
16
14
`x ≅ y`, but previously the three operators in `≡-syntax` unnecessarily require
17
15
`x` and `y` to have the same type, making them unusable in most situations.
18
16
17
+
* Removed unnecessary parameter `#-trans : Transitive _#_` from
18
+
`Relation.Binary.Reasoning.Base.Apartness`.
19
+
19
20
Non-backwards compatible changes
20
21
--------------------------------
21
22
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
-
24
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.
25
24
26
25
* The names exposed by the `IsSemiringWithoutOne` record have been altered to
*[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.
34
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.
35
+
35
36
Minor improvements
36
37
------------------
37
38
@@ -109,16 +110,6 @@ Deprecated names
109
110
New modules
110
111
-----------
111
112
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
-
122
113
* Consequences of module monomorphisms
123
114
```agda
124
115
Algebra.Module.Morphism.BimoduleMonomorphism
@@ -131,6 +122,16 @@ New modules
131
122
Algebra.Module.Morphism.SemimoduleMonomorphism
132
123
```
133
124
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
+
134
135
* Refactoring of the `Algebra.Solver.*Monoid` implementations, via
135
136
a single `Solver` module API based on the existing `Expr`, and
136
137
a common `Normal`-form API:
@@ -144,37 +145,37 @@ New modules
144
145
145
146
NB Imports of the existing proof procedures `solve` and `prove` etc. should still be via the top-level interfaces in `Algebra.Solver.*Monoid`.
146
147
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`
0 commit comments