Skip to content

Commit ff77df9

Browse files
jamesmckinnaandreasabel
authored andcommitted
Spellchecked CHANGELOG (#2078)
1 parent 9cdb0fb commit ff77df9

File tree

1 file changed

+11
-16
lines changed

1 file changed

+11
-16
lines changed

CHANGELOG.md

+11-16
Original file line numberDiff line numberDiff line change
@@ -411,7 +411,7 @@ Non-backwards compatible changes
411411
* At the moment, there are 4 different ways such instance arguments can be provided,
412412
listed in order of convenience and clarity:
413413
1. *Automatic basic instances* - the standard library provides instances based on the constructors of each
414-
numeric type in `Data.X.Base`. For example, `Data.Nat.Base` constains an instance of `NonZero (suc n)` for any `n`
414+
numeric type in `Data.X.Base`. For example, `Data.Nat.Base` constrains an instance of `NonZero (suc n)` for any `n`
415415
and `Data.Integer.Base` contains an instance of `NonNegative (+ n)` for any `n`. Consequently,
416416
if the argument is of the required form, these instances will always be filled in by instance search
417417
automatically, e.g.
@@ -589,7 +589,7 @@ Non-backwards compatible changes
589589
```
590590

591591
* A new module `Reflection.AST` that re-exports the contents of the
592-
submodules has been addeed.
592+
submodules has been added.
593593

594594
### Implementation of division and modulus for ``
595595

@@ -617,7 +617,7 @@ Non-backwards compatible changes
617617
* `IsSemiringWithoutAnnihilatingZero`
618618
* `IsRing`
619619
* To aid with migration, structures matching the old style ones have been added
620-
to `Algebra.Structures.Biased`, with conversionFunctions:
620+
to `Algebra.Structures.Biased`, with conversion functions:
621621
* `IsNearSemiring*` and `isNearSemiring*`
622622
* `IsSemiringWithoutOne*` and `isSemiringWithoutOne*`
623623
* `IsSemiringWithoutAnnihilatingZero*` and `isSemiringWithoutAnnihilatingZero*`
@@ -634,7 +634,7 @@ Non-backwards compatible changes
634634
⊥ = Irrelevant Empty
635635
```
636636
in order to make ⊥ proof irrelevant. Any two proofs of `` or of a negated
637-
statements are now *judgementally* equal to each other.
637+
statements are now *judgmentally* equal to each other.
638638

639639
* Consequently we have modified the following definitions:
640640
+ In `Relation.Nullary.Decidable.Core`, the type of `dec-no` has changed
@@ -671,14 +671,14 @@ Non-backwards compatible changes
671671
however all their contents is re-exported by `Relation.Nullary` which is the easiest way to access
672672
it now.
673673
674-
* In order to facilitate this reorganisation the following breaking moves have occured:
674+
* In order to facilitate this reorganisation the following breaking moves have occurred:
675675
- `¬?` has been moved from `Relation.Nullary.Negation.Core` to `Relation.Nullary.Decidable.Core`
676676
- `¬-reflects` has been moved from `Relation.Nullary.Negation.Core` to `Relation.Nullary.Reflects`.
677677
- `decidable-stable`, `excluded-middle` and `¬-drop-Dec` have been moved from `Relation.Nullary.Negation`
678678
to `Relation.Nullary.Decidable`.
679-
- `fromDec` and `toDec` have been mvoed from `Data.Sum.Base` to `Data.Sum`.
679+
- `fromDec` and `toDec` have been moved from `Data.Sum.Base` to `Data.Sum`.
680680
681-
### Refactoring of the unindexed Functor/Applicative/Monad hiearchy
681+
### Refactoring of the unindexed Functor/Applicative/Monad hierarchy
682682
683683
* The unindexed versions are not defined in terms of the named versions anymore
684684
@@ -698,7 +698,7 @@ Non-backwards compatible changes
698698
699699
* `MonadT T` now returns a `MonadTd` record that packs both a proof that the
700700
`Monad M` transformed by `T` is a monad and that we can `lift` a computation
701-
`M A` to a trasnformed computation `T M A`.
701+
`M A` to a transformed computation `T M A`.
702702
703703
* The monad transformer are not mere aliases anymore, they are record-wrapped
704704
which allows constraints such as `MonadIO (StateT S (ReaderT R IO))` to be
@@ -789,12 +789,12 @@ Non-backwards compatible changes
789789
previous implementation using the sum type `a ⟶ b ⊎ b ⟶ a`.
790790

791791
* In `Algebra.Morphism.Structures`, `IsNearSemiringHomomorphism`,
792-
`IsSemiringHomomorphism`, and `IsRingHomomorphism` have been redeisgned to
792+
`IsSemiringHomomorphism`, and `IsRingHomomorphism` have been redesigned to
793793
build up from `IsMonoidHomomorphism`, `IsNearSemiringHomomorphism`, and
794794
`IsSemiringHomomorphism` respectively, adding a single property at each step.
795795
This means that they no longer need to have two separate proofs of
796796
`IsRelHomomorphism`. Similarly, `IsLatticeHomomorphism` is now built as
797-
`IsRelHomomorphism` along with proofs that `_∧_` and `_∨_` are homorphic.
797+
`IsRelHomomorphism` along with proofs that `_∧_` and `_∨_` are homomorphic.
798798

799799
Also, `⁻¹-homo` in `IsRingHomomorphism` has been renamed to `-‿homo`.
800800

@@ -939,7 +939,7 @@ Major improvements
939939
940940
* To fix this, these operators have been moved to `Data.Nat.Base`. The properties
941941
for them still live in `Data.Nat.DivMod` (which also publicly re-exports them
942-
to provide backwards compatability).
942+
to provide backwards compatibility).
943943
944944
* Beneficiaries of this change include `Data.Rational.Unnormalised.Base` whose
945945
dependencies are now significantly smaller.
@@ -1604,11 +1604,6 @@ New modules
16041604
Data.List.NonEmpty.Relation.Unary.All
16051605
```
16061606

1607-
* A small library for heterogenous equational reasoning on vectors:
1608-
```
1609-
Data.Vec.Properties.Heterogeneous
1610-
```
1611-
16121607
* Show module for unnormalised rationals:
16131608
```
16141609
Data.Rational.Unnormalised.Show

0 commit comments

Comments
 (0)