@@ -539,7 +539,7 @@ Non-backwards compatible changes
539539 3. Finally, if the above approaches are not viable then you may be forced to explicitly
540540 use `cong` combined with a lemma that proves the old reduction behaviour.
541541
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`
543543 has been made into a data type with the single constructor `*≡*`. The destructor `drop-*≡*`
544544 has been added to `Data.Rational.Properties`.
545545
@@ -931,40 +931,40 @@ Non-backwards compatible changes
931931 as would be expected. Instead it omitted several fields like irreflexivity as they were derivable from the
932932 proof of trichotomy. However, this led to problems further up the hierarchy where bundles such as ` StrictTotalOrder `
933933 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.
937937
938938* 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 ` ) .
940940 Therefore the old code:
941941 ``` agda
942942 <-isStrictTotalOrder : IsStrictTotalOrder _≡_ _<_
943943 <-isStrictTotalOrder = record
944- { isEquivalence = isEquivalence
945- ; trans = <-trans
946- ; compare = <-cmp
947- }
944+ { isEquivalence = isEquivalence
945+ ; trans = <-trans
946+ ; compare = <-cmp
947+ }
948948 ```
949949 can be migrated either by updating to the new record fields if you have a proof of ` IsStrictPartialOrder `
950950 available:
951951 ``` agda
952952 <-isStrictTotalOrder : IsStrictTotalOrder _≡_ _<_
953953 <-isStrictTotalOrder = record
954- { isStrictPartialOrder = <-isStrictPartialOrder
955- ; compare = <-cmp
956- }
954+ { isStrictPartialOrder = <-isStrictPartialOrder
955+ ; compare = <-cmp
956+ }
957957 ```
958958 or simply applying the smart constructor to the record definition as follows:
959959 ``` agda
960960 <-isStrictTotalOrder : IsStrictTotalOrder _≡_ _<_
961961 <-isStrictTotalOrder = isStrictTotalOrderᶜ record
962- { isEquivalence = isEquivalence
963- ; trans = <-trans
964- ; compare = <-cmp
965- }
962+ { isEquivalence = isEquivalence
963+ ; trans = <-trans
964+ ; compare = <-cmp
965+ }
966966 ```
967-
967+
968968### Changes to triple reasoning interface
969969
970970* The module ` Relation.Binary.Reasoning.Base.Triple ` now takes an extra proof that the strict
@@ -1231,11 +1231,11 @@ Major improvements
12311231
12321232### More modular design of equational reasoning.
12331233
1234- * Have introduced a new module ` Relation.Binary.Reasoning.Syntax ` which exports
1234+ * Have introduced a new module ` Relation.Binary.Reasoning.Syntax ` which exports
12351235 a range of modules containing pre-existing reasoning combinator syntax.
12361236
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
12391239 (e.g. see ` ∣-Reasoning ` in ` Data.Nat.Divisibility ` )
12401240
12411241Deprecated modules
@@ -1813,7 +1813,7 @@ Deprecated names
18131813 ``` agda
18141814 _↔⟨⟩_ ↦ _≡⟨⟩_
18151815 ```
1816-
1816+
18171817* In ` Foreign.Haskell.Either ` and ` Foreign.Haskell.Pair ` :
18181818 ```
18191819 toForeign ↦ Foreign.Haskell.Coerce.coerce
@@ -2711,7 +2711,7 @@ Additions to existing modules
27112711 toℕ-inverseˡ : Inverseˡ _≡_ _≡_ toℕ fromℕ
27122712 toℕ-inverseʳ : Inverseʳ _≡_ _≡_ toℕ fromℕ
27132713 toℕ-inverseᵇ : Inverseᵇ _≡_ _≡_ toℕ fromℕ
2714-
2714+
27152715 <-asym : Asymmetric _<_
27162716 ```
27172717
@@ -3168,7 +3168,7 @@ Additions to existing modules
31683168 ∀ {m n} → _Respectsʳ_ (_<_ {m} {n}) _≋_
31693169 <-wellFounded : Transitive _≈_ → _≺_ Respectsʳ _≈_ → WellFounded _≺_ →
31703170 ∀ {n} → WellFounded (_<_ {n})
3171- ```
3171+ ```
31723172
31733173* Added new functions in ` Data.Vec.Relation.Unary.Any ` :
31743174 ```
@@ -3195,9 +3195,9 @@ Additions to existing modules
31953195* Added new application operator synonym to ` Function.Bundles ` :
31963196 ``` agda
31973197 _⟨$⟩_ : Func From To → Carrier From → Carrier To
3198- _⟨$⟩_ = Func.to
3198+ _⟨$⟩_ = Func.to
31993199 ```
3200-
3200+
32013201* Added new proofs in ` Function.Construct.Symmetry ` :
32023202 ```
32033203 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
38993899 blockerAll : List Blocker → Blocker
39003900 blockTC : Blocker → TC A
39013901 ```
3902-
3902+
39033903* Added new file ` Relation.Binary.Reasoning.Base.Apartness `
39043904
39053905 This is how to use it:
0 commit comments