Skip to content

Commit 85d1a6b

Browse files
Add Data.List.Relation.Binary.Sublist.Setoid categorical properties (#2385)
* refactor: `variable` declarations and `contradiction` * refactor: one more `contradiction` * left- and right-unit lemmas * left- and right-unit lemmas * `CHANGELOG` * `CHANGELOG` * associativity; fixes #816 * Use cong2 to save rewrites * Make splits for ⊆-assoc exact, simplifying the [] case * Simplify ⊆-assoc not using rewrite * Remove now unused private helper * fix up names and `assoc` orientation; misc. cleanup * new proofs can now move upwards * delegate proofs to `Setoid.Properties` --------- Co-authored-by: Andreas Abel <[email protected]>
1 parent 507fcf8 commit 85d1a6b

File tree

4 files changed

+197
-153
lines changed

4 files changed

+197
-153
lines changed

CHANGELOG.md

+12
Original file line numberDiff line numberDiff line change
@@ -380,6 +380,18 @@ Additions to existing modules
380380
map-catMaybes : map f ∘ catMaybes ≗ catMaybes ∘ map (Maybe.map f)
381381
```
382382

383+
* In `Data.List.Relation.Binary.Sublist.Setoid.Properties`:
384+
```agda
385+
⊆-trans-idˡ : (trans-reflˡ : ∀ {x y} (p : x ≈ y) → trans ≈-refl p ≡ p) →
386+
(pxs : xs ⊆ ys) → ⊆-trans ⊆-refl pxs ≡ pxs
387+
⊆-trans-idʳ : (trans-reflʳ : ∀ {x y} (p : x ≈ y) → trans p ≈-refl ≡ p) →
388+
(pxs : xs ⊆ ys) → ⊆-trans pxs ⊆-refl ≡ pxs
389+
⊆-trans-assoc : (≈-assoc : ∀ {w x y z} (p : w ≈ x) (q : x ≈ y) (r : y ≈ z) →
390+
trans p (trans q r) ≡ trans (trans p q) r) →
391+
(ps : as ⊆ bs) (qs : bs ⊆ cs) (rs : cs ⊆ ds) →
392+
⊆-trans ps (⊆-trans qs rs) ≡ ⊆-trans (⊆-trans ps qs) rs
393+
```
394+
383395
* In `Data.List.Relation.Binary.Subset.Setoid.Properties`:
384396
```agda
385397
map⁺ : f Preserves _≈_ ⟶ _≈′_ → as ⊆ bs → map f as ⊆′ map f bs

0 commit comments

Comments
 (0)