@@ -606,7 +606,7 @@ Non-backwards compatible changes
606
606
* It was very difficult to use the `Relation.Nullary` modules, as `Relation.Nullary`
607
607
contained the basic definitions of negation, decidability etc., and the operations and
608
608
proofs were smeared over `Relation.Nullary.(Negation/Product/Sum/Implication etc.)`.
609
-
609
+
610
610
* In order to fix this:
611
611
- the definition of `Dec` and `recompute` have been moved to `Relation.Nullary.Decidable.Core`
612
612
- the definition of `Reflects` has been moved to `Relation.Nullary.Reflects`
@@ -623,11 +623,11 @@ Non-backwards compatible changes
623
623
have been deprecated and their contents moved to `Relation.Nullary.(Negation/Reflects/Decidable)`
624
624
however all their contents is re-exported by `Relation.Nullary` which is the easiest way to access
625
625
it now.
626
-
626
+
627
627
* In order to facilitate this reorganisation the following breaking moves have occured:
628
628
- `¬?` has been moved from `Relation.Nullary.Negation.Core` to `Relation.Nullary.Decidable.Core`
629
629
- `¬-reflects` has been moved from `Relation.Nullary.Negation.Core` to `Relation.Nullary.Reflects`.
630
- - `decidable-stable`, `excluded-middle` and `¬-drop-Dec` have been moved from `Relation.Nullary.Negation`
630
+ - `decidable-stable`, `excluded-middle` and `¬-drop-Dec` have been moved from `Relation.Nullary.Negation`
631
631
to `Relation.Nullary.Decidable`.
632
632
- `fromDec` and `toDec` have been mvoed from `Data.Sum.Base` to `Data.Sum`.
633
633
@@ -773,7 +773,7 @@ Non-backwards compatible changes
773
773
```
774
774
NB. It is not possible to rename or deprecate ` syntax ` declarations, so Agda will
775
775
only issue a "Could not parse the application ` begin ... ` when scope checking"
776
- warning if the old combinators are used.
776
+ warning if the old combinators are used.
777
777
778
778
* The types of the proofs ` pos⇒1/pos ` /` 1/pos⇒pos ` and ` neg⇒1/neg ` /` 1/neg⇒neg ` in
779
779
` Data.Rational(.Unnormalised).Properties ` have been switched, as the previous
@@ -1073,7 +1073,7 @@ Deprecated names
1073
1073
1074
1074
* In ` Data.Fin.Induction ` :
1075
1075
```
1076
- ≺-Rec
1076
+ ≺-Rec
1077
1077
≺-wellFounded
1078
1078
≺-recBuilder
1079
1079
≺-rec
@@ -1082,7 +1082,7 @@ Deprecated names
1082
1082
As with Issue #1726 above: the deprecation of relation ` _≺_ ` means that these definitions
1083
1083
associated with wf-recursion are deprecated in favour of their ` _<_ ` counterparts.
1084
1084
But it's not quite sensible to say that these definiton should be * renamed* to * anything* ,
1085
- least of all those counterparts... the type confusion would be intolerable.
1085
+ least of all those counterparts... the type confusion would be intolerable.
1086
1086
1087
1087
* In ` Data.Fin.Properties ` :
1088
1088
```
@@ -1163,14 +1163,14 @@ Deprecated names
1163
1163
1164
1164
^-semigroup-morphism ↦ ^-isMagmaHomomorphism
1165
1165
^-monoid-morphism ↦ ^-isMonoidHomomorphism
1166
-
1166
+
1167
1167
pos-distrib-* ↦ pos-*
1168
1168
pos-+-commute ↦ pos-+
1169
1169
abs-*-commute ↦ abs-*
1170
-
1170
+
1171
1171
+-isAbelianGroup ↦ +-0-isAbelianGroup
1172
1172
```
1173
-
1173
+
1174
1174
* In ` Data.List.Properties ` :
1175
1175
``` agda
1176
1176
map-id₂ ↦ map-id-local
@@ -1661,7 +1661,7 @@ New modules
1661
1661
```
1662
1662
Algebra.Properties.Quasigroup
1663
1663
```
1664
-
1664
+
1665
1665
* Properties of MiddleBolLoop
1666
1666
```
1667
1667
Algebra.Properties.MiddleBolLoop
@@ -1828,7 +1828,7 @@ Other minor changes
1828
1828
_MiddleFourExchange_ : Op₂ A → Op₂ A → Set _
1829
1829
1830
1830
SelfInverse : Op₁ A → Set _
1831
-
1831
+
1832
1832
LeftDividesˡ : Op₂ A → Op₂ A → Set _
1833
1833
LeftDividesʳ : Op₂ A → Op₂ A → Set _
1834
1834
RightDividesˡ : Op₂ A → Op₂ A → Set _
@@ -1864,7 +1864,7 @@ Other minor changes
1864
1864
_^ᵗ_ : A → ℕ → A
1865
1865
```
1866
1866
1867
- * ` Algebra.Properties.Magma.Divisibility ` now re-exports operations
1867
+ * ` Algebra.Properties.Magma.Divisibility ` now re-exports operations
1868
1868
` _∣ˡ_ ` , ` _∤ˡ_ ` , ` _∣ʳ_ ` , ` _∤ʳ_ ` from ` Algebra.Definitions.Magma ` .
1869
1869
1870
1870
* Added new proofs to ` Algebra.Properties.CommutativeSemigroup ` :
@@ -2046,7 +2046,7 @@ Other minor changes
2046
2046
* Added new functions in ` Data.Integer.Base ` :
2047
2047
```
2048
2048
_^_ : ℤ → ℕ → ℤ
2049
-
2049
+
2050
2050
+-0-rawGroup : Rawgroup 0ℓ 0ℓ
2051
2051
2052
2052
*-rawMagma : RawMagma 0ℓ 0ℓ
@@ -2164,7 +2164,7 @@ Other minor changes
2164
2164
_! : ℕ → ℕ
2165
2165
2166
2166
parity : ℕ → Parity
2167
-
2167
+
2168
2168
+-rawMagma : RawMagma 0ℓ 0ℓ
2169
2169
+-0-rawMonoid : RawMonoid 0ℓ 0ℓ
2170
2170
*-rawMagma : RawMagma 0ℓ 0ℓ
@@ -2409,10 +2409,10 @@ Other minor changes
2409
2409
* Added new proof to ` Data.Product.Relation.Binary.Lex.Strict `
2410
2410
``` agda
2411
2411
×-respectsʳ : Transitive _≈₁_ →
2412
- _<₁_ Respectsʳ _≈₁_ → _<₂_ Respectsʳ _≈₂_ → _<ₗₑₓ_ Respectsʳ _≋_
2412
+ _<₁_ Respectsʳ _≈₁_ → _<₂_ Respectsʳ _≈₂_ → _<ₗₑₓ_ Respectsʳ _≋_
2413
2413
×-respectsˡ : Symmetric _≈₁_ → Transitive _≈₁_ →
2414
- _<₁_ Respectsˡ _≈₁_ → _<₂_ Respectsˡ _≈₂_ → _<ₗₑₓ_ Respectsˡ _≋_
2415
- ×-wellFounded' : Symmetric _≈₁_ → Transitive _≈₁_ → _<₁_ Respectsʳ _≈₁_ →
2414
+ _<₁_ Respectsˡ _≈₁_ → _<₂_ Respectsˡ _≈₂_ → _<ₗₑₓ_ Respectsˡ _≋_
2415
+ ×-wellFounded' : Symmetric _≈₁_ → Transitive _≈₁_ → _<₁_ Respectsʳ _≈₁_ →
2416
2416
WellFounded _<₁_ → WellFounded _<₂_ → WellFounded _<ₗₑₓ_
2417
2417
```
2418
2418
@@ -2565,7 +2565,7 @@ Other minor changes
2565
2565
∀ {m n} → _Respectsˡ_ (_<_ {m} {n}) _≋_
2566
2566
<-respectsʳ : IsPartialEquivalence _≈_ → _≺_ Respectsʳ _≈_ →
2567
2567
∀ {m n} → _Respectsʳ_ (_<_ {m} {n}) _≋_
2568
- <-wellFounded : Symmetric _≈_ → Transitive _≈_ → _≺_ Respectsʳ _≈_ → WellFounded _≺_ →
2568
+ <-wellFounded : Symmetric _≈_ → Transitive _≈_ → _≺_ Respectsʳ _≈_ → WellFounded _≺_ →
2569
2569
∀ {n} → WellFounded (_<_ {n})
2570
2570
```
2571
2571
@@ -3184,14 +3184,21 @@ This is a full list of proofs that have changed form to use irrelevant instance
3184
3184
↭-reverse : (xs : List A) → reverse xs ↭ xs
3185
3185
```
3186
3186
3187
- * Added new file ` Relation.Binary.Reasoning.Base.Apartness `
3188
-
3189
- This is how to use it:
3187
+ * Added new proofs to ` Data.List.Relation.Binary.Sublist.Setoid.Properties `
3188
+ and ` Data.List.Relation.Unary.Sorted.TotalOrder.Properties ` .
3190
3189
``` agda
3191
- _ : a # d
3192
- _ = begin-apartness
3193
- a ≈⟨ a≈b ⟩
3194
- b #⟨ b#c ⟩
3195
- c ≈⟨ c≈d ⟩
3196
- d ∎
3190
+ ⊆-mergeˡ : ∀ xs ys → xs ⊆ merge _≤?_ xs ys
3191
+ ⊆-mergeʳ : ∀ xs ys → ys ⊆ merge _≤?_ xs ys
3197
3192
```
3193
+
3194
+ * Added new file ` Relation.Binary.Reasoning.Base.Apartness `
3195
+
3196
+ This is how to use it:
3197
+ ``` agda
3198
+ _ : a # d
3199
+ _ = begin-apartness
3200
+ a ≈⟨ a≈b ⟩
3201
+ b #⟨ b#c ⟩
3202
+ c ≈⟨ c≈d ⟩
3203
+ d ∎
3204
+ ```
0 commit comments