@@ -112,21 +112,21 @@ Non-backwards compatible changes
112
112
always true and cannot be assumed in user's code.
113
113
114
114
* Therefore the definitions have been changed as follows to make all their arguments explicit:
115
- - ` LeftCancellative _• _ `
116
- - From: ` ∀ x {y z} → (x • y) ≈ (x • z) → y ≈ z `
117
- - To: ` ∀ x y z → (x • y) ≈ (x • z) → y ≈ z `
115
+ - ` LeftCancellative _∙ _ `
116
+ - From: ` ∀ x {y z} → (x ∙ y) ≈ (x ∙ z) → y ≈ z `
117
+ - To: ` ∀ x y z → (x ∙ y) ≈ (x ∙ z) → y ≈ z `
118
118
119
- - ` RightCancellative _• _ `
120
- - From: ` ∀ {x} y z → (y • x) ≈ (z • x) → y ≈ z `
121
- - To: ` ∀ x y z → (y • x) ≈ (z • x) → y ≈ z `
119
+ - ` RightCancellative _∙ _ `
120
+ - From: ` ∀ {x} y z → (y ∙ x) ≈ (z ∙ x) → y ≈ z `
121
+ - To: ` ∀ x y z → (y ∙ x) ≈ (z ∙ x) → y ≈ z `
122
122
123
- - ` AlmostLeftCancellative e _• _ `
124
- - From: ` ∀ {x} y z → ¬ x ≈ e → (x • y) ≈ (x • z) → y ≈ z `
125
- - To: ` ∀ x y z → ¬ x ≈ e → (x • y) ≈ (x • z) → y ≈ z `
123
+ - ` AlmostLeftCancellative e _∙ _ `
124
+ - From: ` ∀ {x} y z → ¬ x ≈ e → (x ∙ y) ≈ (x ∙ z) → y ≈ z `
125
+ - To: ` ∀ x y z → ¬ x ≈ e → (x ∙ y) ≈ (x ∙ z) → y ≈ z `
126
126
127
- - ` AlmostRightCancellative e _• _ `
128
- - From: ` ∀ {x} y z → ¬ x ≈ e → (y • x) ≈ (z • x) → y ≈ z `
129
- - To: ` ∀ x y z → ¬ x ≈ e → (y • x) ≈ (z • x) → y ≈ z `
127
+ - ` AlmostRightCancellative e _∙ _ `
128
+ - From: ` ∀ {x} y z → ¬ x ≈ e → (y ∙ x) ≈ (z ∙ x) → y ≈ z `
129
+ - To: ` ∀ x y z → ¬ x ≈ e → (y ∙ x) ≈ (z ∙ x) → y ≈ z `
130
130
131
131
* Correspondingly some proofs of the above types will need additional arguments passed explicitly.
132
132
Instances can easily be fixed by adding additional underscores, e.g.
@@ -2152,16 +2152,16 @@ Additions to existing modules
2152
2152
2153
2153
* Added new proofs to ` Algebra.Consequences.Propositional ` :
2154
2154
``` agda
2155
- comm+assoc⇒middleFour : Commutative _• _ → Associative _• _ → _• _ MiddleFourExchange _• _
2156
- identity+middleFour⇒assoc : Identity e _• _ → _• _ MiddleFourExchange _• _ → Associative _• _
2157
- identity+middleFour⇒comm : Identity e _+_ → _• _ MiddleFourExchange _+_ → Commutative _• _
2155
+ comm+assoc⇒middleFour : Commutative _∙ _ → Associative _∙ _ → _∙ _ MiddleFourExchange _∙ _
2156
+ identity+middleFour⇒assoc : Identity e _∙ _ → _∙ _ MiddleFourExchange _∙ _ → Associative _∙ _
2157
+ identity+middleFour⇒comm : Identity e _+_ → _∙ _ MiddleFourExchange _+_ → Commutative _∙ _
2158
2158
```
2159
2159
2160
2160
* Added new proofs to ` Algebra.Consequences.Setoid ` :
2161
2161
``` agda
2162
- comm+assoc⇒middleFour : Congruent₂ _• _ → Commutative _• _ → Associative _• _ → _• _ MiddleFourExchange _• _
2163
- identity+middleFour⇒assoc : Congruent₂ _• _ → Identity e _• _ → _• _ MiddleFourExchange _• _ → Associative _• _
2164
- identity+middleFour⇒comm : Congruent₂ _• _ → Identity e _+_ → _• _ MiddleFourExchange _+_ → Commutative _• _
2162
+ comm+assoc⇒middleFour : Congruent₂ _∙ _ → Commutative _∙ _ → Associative _∙ _ → _∙ _ MiddleFourExchange _∙ _
2163
+ identity+middleFour⇒assoc : Congruent₂ _∙ _ → Identity e _∙ _ → _∙ _ MiddleFourExchange _∙ _ → Associative _∙ _
2164
+ identity+middleFour⇒comm : Congruent₂ _∙ _ → Identity e _+_ → _∙ _ MiddleFourExchange _+_ → Commutative _∙ _
2165
2165
2166
2166
involutive⇒surjective : Involutive f → Surjective f
2167
2167
selfInverse⇒involutive : SelfInverse f → Involutive f
@@ -2171,15 +2171,15 @@ Additions to existing modules
2171
2171
selfInverse⇒injective : SelfInverse f → Injective f
2172
2172
selfInverse⇒bijective : SelfInverse f → Bijective f
2173
2173
2174
- comm+idˡ⇒id : Commutative _• _ → LeftIdentity e _• _ → Identity e _• _
2175
- comm+idʳ⇒id : Commutative _• _ → RightIdentity e _• _ → Identity e _• _
2176
- comm+zeˡ⇒ze : Commutative _• _ → LeftZero e _• _ → Zero e _• _
2177
- comm+zeʳ⇒ze : Commutative _• _ → RightZero e _• _ → Zero e _• _
2178
- comm+invˡ⇒inv : Commutative _• _ → LeftInverse e _⁻¹ _• _ → Inverse e _⁻¹ _• _
2179
- comm+invʳ⇒inv : Commutative _• _ → RightInverse e _⁻¹ _• _ → Inverse e _⁻¹ _• _
2180
- comm+distrˡ⇒distr : Commutative _• _ → _• _ DistributesOverˡ _◦_ → _• _ DistributesOver _◦_
2181
- comm+distrʳ⇒distr : Commutative _• _ → _• _ DistributesOverʳ _◦_ → _• _ DistributesOver _◦_
2182
- distrib+absorbs⇒distribˡ : Associative _• _ → Commutative _◦_ → _• _ Absorbs _◦_ → _◦_ Absorbs _• _ → _◦_ DistributesOver _• _ → _• _ DistributesOverˡ _◦_
2174
+ comm+idˡ⇒id : Commutative _∙ _ → LeftIdentity e _∙ _ → Identity e _∙ _
2175
+ comm+idʳ⇒id : Commutative _∙ _ → RightIdentity e _∙ _ → Identity e _∙ _
2176
+ comm+zeˡ⇒ze : Commutative _∙ _ → LeftZero e _∙ _ → Zero e _∙ _
2177
+ comm+zeʳ⇒ze : Commutative _∙ _ → RightZero e _∙ _ → Zero e _∙ _
2178
+ comm+invˡ⇒inv : Commutative _∙ _ → LeftInverse e _⁻¹ _∙ _ → Inverse e _⁻¹ _∙ _
2179
+ comm+invʳ⇒inv : Commutative _∙ _ → RightInverse e _⁻¹ _∙ _ → Inverse e _⁻¹ _∙ _
2180
+ comm+distrˡ⇒distr : Commutative _∙ _ → _∙ _ DistributesOverˡ _◦_ → _∙ _ DistributesOver _◦_
2181
+ comm+distrʳ⇒distr : Commutative _∙ _ → _∙ _ DistributesOverʳ _◦_ → _∙ _ DistributesOver _◦_
2182
+ distrib+absorbs⇒distribˡ : Associative _∙ _ → Commutative _◦_ → _∙ _ Absorbs _◦_ → _◦_ Absorbs _∙ _ → _◦_ DistributesOver _∙ _ → _∙ _ DistributesOverˡ _◦_
2183
2183
```
2184
2184
2185
2185
* Added new functions to ` Algebra.Construct.DirectProduct ` :
0 commit comments