@@ -141,28 +141,28 @@ Additions to existing modules
141
141
142
142
* In ` Data.List.Relation.Ternary.Appending.Setoid.Properties ` :
143
143
``` agda
144
- through→ : ∃[ xs ] Pointwise _≈_ as xs × Appending xs bs cs →
144
+ through→ : ∃[ xs ] Pointwise _≈_ as xs × Appending xs bs cs →
145
145
∃[ ys ] Appending as bs ys × Pointwise _≈_ ys cs
146
- through← : ∃[ ys ] Appending as bs ys × Pointwise _≈_ ys cs →
146
+ through← : ∃[ ys ] Appending as bs ys × Pointwise _≈_ ys cs →
147
147
∃[ xs ] Pointwise _≈_ as xs × Appending xs bs cs
148
- assoc→ : ∃[ xs ] Appending as bs xs × Appending xs cs ds →
148
+ assoc→ : ∃[ xs ] Appending as bs xs × Appending xs cs ds →
149
149
∃[ ys ] Appending bs cs ys × Appending as ys ds
150
150
```
151
151
152
152
* In ` Data.List.Relation.Ternary.Appending.Properties ` :
153
153
``` agda
154
- through→ : (R ⇒ (S ; T)) → ((U ; V) ⇒ (W ; T)) →
155
- ∃[ xs ] Pointwise U as xs × Appending V R xs bs cs →
156
- ∃[ ys ] Appending W S as bs ys × Pointwise T ys cs
157
- through← : ((R ; S) ⇒ T) → ((U ; S) ⇒ (V ; W)) →
158
- ∃[ ys ] Appending U R as bs ys × Pointwise S ys cs →
159
- ∃[ xs ] Pointwise V as xs × Appending W T xs bs cs
160
- assoc→ : (R ⇒ (S ; T)) → ((U ; V) ⇒ (W ; T)) → ((Y ; V) ⇒ X) →
161
- ∃[ xs ] Appending Y U as bs xs × Appending V R xs cs ds →
162
- ∃[ ys ] Appending W S bs cs ys × Appending X T as ys ds
163
- assoc← : ((S ; T) ⇒ R) → ((W ; T) ⇒ (U ; V)) → (X ⇒ (Y ; V)) →
164
- ∃[ ys ] Appending W S bs cs ys × Appending X T as ys ds →
165
- ∃[ xs ] Appending Y U as bs xs × Appending V R xs cs ds
154
+ through→ : (R ⇒ (S ; T)) → ((U ; V) ⇒ (W ; T)) →
155
+ ∃[ xs ] Pointwise U as xs × Appending V R xs bs cs →
156
+ ∃[ ys ] Appending W S as bs ys × Pointwise T ys cs
157
+ through← : ((R ; S) ⇒ T) → ((U ; S) ⇒ (V ; W)) →
158
+ ∃[ ys ] Appending U R as bs ys × Pointwise S ys cs →
159
+ ∃[ xs ] Pointwise V as xs × Appending W T xs bs cs
160
+ assoc→ : (R ⇒ (S ; T)) → ((U ; V) ⇒ (W ; T)) → ((Y ; V) ⇒ X) →
161
+ ∃[ xs ] Appending Y U as bs xs × Appending V R xs cs ds →
162
+ ∃[ ys ] Appending W S bs cs ys × Appending X T as ys ds
163
+ assoc← : ((S ; T) ⇒ R) → ((W ; T) ⇒ (U ; V)) → (X ⇒ (Y ; V)) →
164
+ ∃[ ys ] Appending W S bs cs ys × Appending X T as ys ds →
165
+ ∃[ xs ] Appending Y U as bs xs × Appending V R xs cs ds
166
166
```
167
167
168
168
* In ` Data.List.Relation.Binary.Pointwise.Base ` :
@@ -210,6 +210,11 @@ Additions to existing modules
210
210
* In ` Function.Bundles ` , added ` _⟶ₛ_ ` as a synonym for ` Func ` that can
211
211
be used infix.
212
212
213
+ * Added new proofs in ` Relation.Binary.Construct.Composition ` :
214
+ ``` agda
215
+ transitive⇒≈;≈⊆≈ : Transitive ≈ → (≈ ; ≈) ⇒ ≈
216
+ ```
217
+
213
218
* Added new definitions in ` Relation.Binary.Definitions `
214
219
```
215
220
Stable _∼_ = ∀ x y → Nullary.Stable (x ∼ y)
0 commit comments