@@ -411,7 +411,7 @@ Non-backwards compatible changes
411
411
* At the moment, there are 4 different ways such instance arguments can be provided,
412
412
listed in order of convenience and clarity:
413
413
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 `
415
415
and ` Data.Integer.Base ` contains an instance of ` NonNegative (+ n) ` for any ` n ` . Consequently,
416
416
if the argument is of the required form, these instances will always be filled in by instance search
417
417
automatically, e.g.
@@ -589,7 +589,7 @@ Non-backwards compatible changes
589
589
```
590
590
591
591
* A new module ` Reflection.AST ` that re-exports the contents of the
592
- submodules has been addeed .
592
+ submodules has been added .
593
593
594
594
### Implementation of division and modulus for ` ℤ `
595
595
@@ -617,7 +617,7 @@ Non-backwards compatible changes
617
617
* ` IsSemiringWithoutAnnihilatingZero `
618
618
* ` IsRing `
619
619
* 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 :
621
621
* ` IsNearSemiring* ` and ` isNearSemiring* `
622
622
* ` IsSemiringWithoutOne* ` and ` isSemiringWithoutOne* `
623
623
* ` IsSemiringWithoutAnnihilatingZero* ` and ` isSemiringWithoutAnnihilatingZero* `
@@ -634,7 +634,7 @@ Non-backwards compatible changes
634
634
⊥ = Irrelevant Empty
635
635
```
636
636
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.
638
638
639
639
* Consequently we have modified the following definitions:
640
640
+ In ` Relation.Nullary.Decidable.Core ` , the type of ` dec-no ` has changed
@@ -671,14 +671,14 @@ Non-backwards compatible changes
671
671
however all their contents is re-exported by `Relation.Nullary` which is the easiest way to access
672
672
it now.
673
673
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 :
675
675
- `¬?` has been moved from `Relation.Nullary.Negation.Core` to `Relation.Nullary.Decidable.Core`
676
676
- `¬-reflects` has been moved from `Relation.Nullary.Negation.Core` to `Relation.Nullary.Reflects`.
677
677
- `decidable-stable`, `excluded-middle` and `¬-drop-Dec` have been moved from `Relation.Nullary.Negation`
678
678
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`.
680
680
681
- ### Refactoring of the unindexed Functor/Applicative/Monad hiearchy
681
+ ### Refactoring of the unindexed Functor/Applicative/Monad hierarchy
682
682
683
683
* The unindexed versions are not defined in terms of the named versions anymore
684
684
@@ -698,7 +698,7 @@ Non-backwards compatible changes
698
698
699
699
* `MonadT T` now returns a `MonadTd` record that packs both a proof that the
700
700
`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`.
702
702
703
703
* The monad transformer are not mere aliases anymore, they are record-wrapped
704
704
which allows constraints such as `MonadIO (StateT S (ReaderT R IO))` to be
@@ -789,12 +789,12 @@ Non-backwards compatible changes
789
789
previous implementation using the sum type ` a ⟶ b ⊎ b ⟶ a ` .
790
790
791
791
* In ` Algebra.Morphism.Structures ` , ` IsNearSemiringHomomorphism ` ,
792
- ` IsSemiringHomomorphism ` , and ` IsRingHomomorphism ` have been redeisgned to
792
+ ` IsSemiringHomomorphism ` , and ` IsRingHomomorphism ` have been redesigned to
793
793
build up from ` IsMonoidHomomorphism ` , ` IsNearSemiringHomomorphism ` , and
794
794
` IsSemiringHomomorphism ` respectively, adding a single property at each step.
795
795
This means that they no longer need to have two separate proofs of
796
796
` 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 .
798
798
799
799
Also, ` ⁻¹-homo ` in ` IsRingHomomorphism ` has been renamed to ` -‿homo ` .
800
800
@@ -939,7 +939,7 @@ Major improvements
939
939
940
940
* To fix this, these operators have been moved to `Data.Nat.Base`. The properties
941
941
for them still live in `Data.Nat.DivMod` (which also publicly re-exports them
942
- to provide backwards compatability ).
942
+ to provide backwards compatibility ).
943
943
944
944
* Beneficiaries of this change include `Data.Rational.Unnormalised.Base` whose
945
945
dependencies are now significantly smaller.
@@ -1604,11 +1604,6 @@ New modules
1604
1604
Data.List.NonEmpty.Relation.Unary.All
1605
1605
```
1606
1606
1607
- * A small library for heterogenous equational reasoning on vectors:
1608
- ```
1609
- Data.Vec.Properties.Heterogeneous
1610
- ```
1611
-
1612
1607
* Show module for unnormalised rationals:
1613
1608
```
1614
1609
Data.Rational.Unnormalised.Show
0 commit comments