Skip to content

Commit fcef696

Browse files
More minor tweaks to the CHANGELOG
1 parent daf22fd commit fcef696

File tree

1 file changed

+22
-21
lines changed

1 file changed

+22
-21
lines changed

CHANGELOG.md

Lines changed: 22 additions & 21 deletions
Original file line numberDiff line numberDiff line change
@@ -45,7 +45,7 @@ Non-backwards compatible changes
4545
affect users who are renaming/hiding the library's equational reasoning combinators.
4646

4747
* Previously all equational reasoning combinators (e.g. `_≈⟨_⟩_`, `_≡⟨_⟩_`, `_≤⟨_⟩_`)
48-
have been defined in the following style:
48+
were defined in the following style:
4949
```agda
5050
infixr 2 _≡⟨_⟩_
5151
@@ -83,8 +83,9 @@ Non-backwards compatible changes
8383
compatible. Having said that you may want to switch to the new style for the benefits
8484
described above.
8585

86-
* **Changes required**: The one drawback is that hiding and renaming the combinators no longer works
87-
as before, as `_≡⟨_⟩_` etc. are now syntax instead of names. For example instead of:
86+
* **Changes required**: The only drawback to this change is that hiding and renaming the
87+
combinators no longer works as before, as `_≡⟨_⟩_` etc. are now syntax instead of names.
88+
For example instead of:
8889
```agda
8990
open SetoidReasoning setoid public
9091
hiding (_≈⟨_⟩_) renaming (_≡⟨_⟩_ to _↭⟨_⟩_)
@@ -110,17 +111,18 @@ Non-backwards compatible changes
110111
- `IsCommutativeMonoid`
111112
- `IsCommutativeSemiring`
112113
- `IsRing`
113-
In all of these cases, the change has been to give each of these structures
114-
access to *all* of the fields of structures below (weaker) in the hierarchy.
115114

116-
* For example, consider `IsCommutativeMonoid`. The old definition effectively
117-
required the following fields.
118-
115+
In each case, the structure now requires fields for all the required properties,
116+
rather than just an (arbitrary) minimal set of properties.
117+
118+
* For example, whereas the old definition of `IsCommutativeMonoid` required
119+
the following fields:
120+
119121
- Associativity
120122
- Left identity
121123
- Commutativity
122124

123-
The new definition also requires:
125+
the new definition also requires:
124126

125127
- Right identity.
126128

@@ -229,8 +231,7 @@ Deprecated modules
229231
The following modules have been renamed as part of a drive to improve
230232
consistency across the library. The deprecated modules still exist and
231233
therefore all existing code should still work, however use of the new names
232-
is encouraged. Automated warnings are attached to deprecated modules to
233-
discourage their use.
234+
is encouraged.
234235

235236
* In `Algebra`:
236237
```
@@ -276,7 +277,7 @@ attached to all deprecated names to discourage their use.
276277
Any¬→¬All ↦ Any¬⇒¬All
277278
```
278279

279-
* In `Data.Nat.Properties
280+
* In `Data.Nat.Properties`:
280281
```agda
281282
∀[m≤n⇒m≢o]⇒o<n ↦ ∀[m≤n⇒m≢o]⇒n<o
282283
∀[m<n⇒m≢o]⇒o≤n ↦ ∀[m<n⇒m≢o]⇒n≤o
@@ -304,7 +305,7 @@ New modules
304305
Algebra.Module.Structures
305306
Algebra.Module.Structures.Biased
306307
```
307-
Supported are all of {left ,right , bi,}{semi,}modules.
308+
Supported are all of {left, right, bi} {semi} modules.
308309

309310
* Morphisms over group and ring-like algebraic structures:
310311
```agda
@@ -356,14 +357,15 @@ New modules
356357
Data.Tree.Rose
357358
Data.Tree.Rose.Properties
358359
```
359-
360+
361+
* New properties and functions over floats and words.
360362
```agda
361363
Data.Float.Base
362364
Data.Float.Properties
363365
Data.Word.Base
364366
Data.Word.Properties
365367
```
366-
368+
367369
* Helper methods for using reflection with numeric data.
368370
```agda
369371
Data.Nat.Reflection
@@ -399,14 +401,13 @@ Other major changes
399401

400402
#### Improved performance of decision processes
401403

402-
* Rewrote definitions branching on a `Dec` value to branch only on the boolean
403-
`does` field, wherever possible. Furthermore, branching on the `proof` field
404-
has been made as late as possible, using the `invert` lemma from
404+
* All definitions branching on a `Dec` value have been rewritten, wherever possible,
405+
to branch only on the boolean `does` field. Furthermore, branching on
406+
the `proof` field has been made as late as possible, using the `invert` lemma from
405407
`Relation.Nullary.Reflects`.
406408

407409
* For example, the old definition of `filter` in `Data.List.Base` used the
408-
`yes` and `no` patterns, which desugared to the following.
409-
410+
`yes` and `no` patterns, which desugared to the following:
410411
```agda
411412
filter : ∀ {P : Pred A p} → Decidable P → List A → List A
412413
filter P? [] = []
@@ -449,7 +450,7 @@ Other major changes
449450

450451
#### Other
451452

452-
* The module `Reflection` is no longer unsafe.
453+
* The module `Reflection` is no longer `--unsafe`.
453454

454455
* Standardised the `Eq` modules in structures and bundles in `Relation.Binary` hierarchy.
455456
- `IsDecTotalOrder.Eq` now exports `isDecPartialOrder`.

0 commit comments

Comments
 (0)