@@ -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
@@ -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
@@ -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
@@ -2711,7 +2711,7 @@ Additions to existing modules
2711
2711
toℕ-inverseˡ : Inverseˡ _≡_ _≡_ toℕ fromℕ
2712
2712
toℕ-inverseʳ : Inverseʳ _≡_ _≡_ toℕ fromℕ
2713
2713
toℕ-inverseᵇ : Inverseᵇ _≡_ _≡_ toℕ fromℕ
2714
-
2714
+
2715
2715
<-asym : Asymmetric _<_
2716
2716
```
2717
2717
@@ -3168,7 +3168,7 @@ Additions to existing modules
3168
3168
∀ {m n} → _Respectsʳ_ (_<_ {m} {n}) _≋_
3169
3169
<-wellFounded : Transitive _≈_ → _≺_ Respectsʳ _≈_ → WellFounded _≺_ →
3170
3170
∀ {n} → WellFounded (_<_ {n})
3171
- ```
3171
+ ```
3172
3172
3173
3173
* Added new functions in ` Data.Vec.Relation.Unary.Any ` :
3174
3174
```
@@ -3195,9 +3195,9 @@ Additions to existing modules
3195
3195
* Added new application operator synonym to ` Function.Bundles ` :
3196
3196
``` agda
3197
3197
_⟨$⟩_ : Func From To → Carrier From → Carrier To
3198
- _⟨$⟩_ = Func.to
3198
+ _⟨$⟩_ = Func.to
3199
3199
```
3200
-
3200
+
3201
3201
* Added new proofs in ` Function.Construct.Symmetry ` :
3202
3202
```
3203
3203
bijective : Bijective ≈₁ ≈₂ f → Symmetric ≈₂ → Transitive ≈₂ → Congruent ≈₁ ≈₂ f → Bijective ≈₂ ≈₁ f⁻¹
@@ -3899,7 +3899,7 @@ This is a full list of proofs that have changed form to use irrelevant instance
3899
3899
blockerAll : List Blocker → Blocker
3900
3900
blockTC : Blocker → TC A
3901
3901
```
3902
-
3902
+
3903
3903
* Added new file ` Relation.Binary.Reasoning.Base.Apartness `
3904
3904
3905
3905
This is how to use it:
0 commit comments