@@ -539,7 +539,7 @@ Non-backwards compatible changes
539
539
3. Finally, if the above approaches are not viable then you may be forced to explicitly
540
540
use `cong` combined with a lemma that proves the old reduction behaviour.
541
541
542
- * Similarly, in order to prevent reduction, the equality `_≃_` in `Data.Rational.Base`
542
+ * Similarly, in order to prevent reduction, the equality `_≃_` in `Data.Rational.Base`
543
543
has been made into a data type with the single constructor `*≡*`. The destructor `drop-*≡*`
544
544
has been added to `Data.Rational.Properties`.
545
545
@@ -606,7 +606,7 @@ Non-backwards compatible changes
606
606
with the consequence that all arguments involving about accesibility and
607
607
wellfoundedness proofs were polluted by almost-always-inferrable explicit
608
608
arguments for the ` y ` position. The definition has now been changed to
609
- make that argument * implicit* , as
609
+ make that argument * implicit* , as
610
610
``` agda
611
611
WfRec : Rel A r → ∀ {ℓ} → RecStruct A ℓ _
612
612
WfRec _<_ P x = ∀ {y} → y < x → P y
@@ -931,40 +931,40 @@ Non-backwards compatible changes
931
931
as would be expected. Instead it omitted several fields like irreflexivity as they were derivable from the
932
932
proof of trichotomy. However, this led to problems further up the hierarchy where bundles such as ` StrictTotalOrder `
933
933
which contained multiple distinct proofs of ` IsStrictPartialOrder ` .
934
-
935
- * To remedy this the definition of ` IsStrictTotalOrder ` has been changed to so that it builds upon
936
- ` IsStrictPartialOrder ` as would be expected.
934
+
935
+ * To remedy this the definition of ` IsStrictTotalOrder ` has been changed to so that it builds upon
936
+ ` IsStrictPartialOrder ` as would be expected.
937
937
938
938
* To aid migration, the old record definition has been moved to ` Relation.Binary.Structures.Biased `
939
- which contains the ` isStrictTotalOrderᶜ ` smart constructor (which is re-exported by ` Relation.Binary ` ) .
939
+ which contains the ` isStrictTotalOrderᶜ ` smart constructor (which is re-exported by ` Relation.Binary ` ) .
940
940
Therefore the old code:
941
941
``` agda
942
942
<-isStrictTotalOrder : IsStrictTotalOrder _≡_ _<_
943
943
<-isStrictTotalOrder = record
944
- { isEquivalence = isEquivalence
945
- ; trans = <-trans
946
- ; compare = <-cmp
947
- }
944
+ { isEquivalence = isEquivalence
945
+ ; trans = <-trans
946
+ ; compare = <-cmp
947
+ }
948
948
```
949
949
can be migrated either by updating to the new record fields if you have a proof of ` IsStrictPartialOrder `
950
950
available:
951
951
``` agda
952
952
<-isStrictTotalOrder : IsStrictTotalOrder _≡_ _<_
953
953
<-isStrictTotalOrder = record
954
- { isStrictPartialOrder = <-isStrictPartialOrder
955
- ; compare = <-cmp
956
- }
954
+ { isStrictPartialOrder = <-isStrictPartialOrder
955
+ ; compare = <-cmp
956
+ }
957
957
```
958
958
or simply applying the smart constructor to the record definition as follows:
959
959
``` agda
960
960
<-isStrictTotalOrder : IsStrictTotalOrder _≡_ _<_
961
961
<-isStrictTotalOrder = isStrictTotalOrderᶜ record
962
- { isEquivalence = isEquivalence
963
- ; trans = <-trans
964
- ; compare = <-cmp
965
- }
962
+ { isEquivalence = isEquivalence
963
+ ; trans = <-trans
964
+ ; compare = <-cmp
965
+ }
966
966
```
967
-
967
+
968
968
### Changes to triple reasoning interface
969
969
970
970
* The module ` Relation.Binary.Reasoning.Base.Triple ` now takes an extra proof that the strict
@@ -987,7 +987,7 @@ Non-backwards compatible changes
987
987
Data.Vec.Relation.Binary.Lex.NonStrict
988
988
Relation.Binary.Reasoning.StrictPartialOrder
989
989
Relation.Binary.Reasoning.PartialOrder
990
- ```
990
+ ```
991
991
992
992
### Other
993
993
@@ -1165,7 +1165,7 @@ Non-backwards compatible changes
1165
1165
* ` excluded-middle ` in ` Relation.Nullary.Decidable.Core ` has been renamed to
1166
1166
` ¬¬-excluded-middle ` .
1167
1167
1168
- * ` iterate ` and ` replicate ` in ` Data.Vec.Base ` and ` Data.Vec.Functional `
1168
+ * ` iterate ` and ` replicate ` in ` Data.Vec.Base ` and ` Data.Vec.Functional `
1169
1169
now take the length of vector, ` n ` , as an explicit rather than an implicit argument.
1170
1170
``` agda
1171
1171
iterate : (A → A) → A → ∀ n → Vec A n
@@ -1231,11 +1231,11 @@ Major improvements
1231
1231
1232
1232
### More modular design of equational reasoning.
1233
1233
1234
- * Have introduced a new module ` Relation.Binary.Reasoning.Syntax ` which exports
1234
+ * Have introduced a new module ` Relation.Binary.Reasoning.Syntax ` which exports
1235
1235
a range of modules containing pre-existing reasoning combinator syntax.
1236
1236
1237
- * This makes it possible to add new or rename existing reasoning combinators to a
1238
- pre-existing ` Reasoning ` module in just a couple of lines
1237
+ * This makes it possible to add new or rename existing reasoning combinators to a
1238
+ pre-existing ` Reasoning ` module in just a couple of lines
1239
1239
(e.g. see ` ∣-Reasoning ` in ` Data.Nat.Divisibility ` )
1240
1240
1241
1241
Deprecated modules
@@ -1813,7 +1813,7 @@ Deprecated names
1813
1813
``` agda
1814
1814
_↔⟨⟩_ ↦ _≡⟨⟩_
1815
1815
```
1816
-
1816
+
1817
1817
* In ` Foreign.Haskell.Either ` and ` Foreign.Haskell.Pair ` :
1818
1818
```
1819
1819
toForeign ↦ Foreign.Haskell.Coerce.coerce
@@ -2706,7 +2706,7 @@ Additions to existing modules
2706
2706
toℕ-inverseˡ : Inverseˡ _≡_ _≡_ toℕ fromℕ
2707
2707
toℕ-inverseʳ : Inverseʳ _≡_ _≡_ toℕ fromℕ
2708
2708
toℕ-inverseᵇ : Inverseᵇ _≡_ _≡_ toℕ fromℕ
2709
-
2709
+
2710
2710
<-asym : Asymmetric _<_
2711
2711
```
2712
2712
@@ -3163,7 +3163,7 @@ Additions to existing modules
3163
3163
∀ {m n} → _Respectsʳ_ (_<_ {m} {n}) _≋_
3164
3164
<-wellFounded : Transitive _≈_ → _≺_ Respectsʳ _≈_ → WellFounded _≺_ →
3165
3165
∀ {n} → WellFounded (_<_ {n})
3166
- ```
3166
+ ```
3167
3167
3168
3168
* Added new functions in ` Data.Vec.Relation.Unary.Any ` :
3169
3169
```
@@ -3190,9 +3190,9 @@ Additions to existing modules
3190
3190
* Added new application operator synonym to ` Function.Bundles ` :
3191
3191
``` agda
3192
3192
_⟨$⟩_ : Func From To → Carrier From → Carrier To
3193
- _⟨$⟩_ = Func.to
3193
+ _⟨$⟩_ = Func.to
3194
3194
```
3195
-
3195
+
3196
3196
* Added new proofs in ` Function.Construct.Symmetry ` :
3197
3197
```
3198
3198
bijective : Bijective ≈₁ ≈₂ f → Symmetric ≈₂ → Transitive ≈₂ → Congruent ≈₁ ≈₂ f → Bijective ≈₂ ≈₁ f⁻¹
@@ -3888,7 +3888,7 @@ This is a full list of proofs that have changed form to use irrelevant instance
3888
3888
blockerAll : List Blocker → Blocker
3889
3889
blockTC : Blocker → TC A
3890
3890
```
3891
-
3891
+
3892
3892
* Added new file ` Relation.Binary.Reasoning.Base.Apartness `
3893
3893
3894
3894
This is how to use it:
0 commit comments