File tree Expand file tree Collapse file tree 3 files changed +26
-0
lines changed
src/Data/List/Relation/Binary/Subset Expand file tree Collapse file tree 3 files changed +26
-0
lines changed Original file line number Diff line number Diff line change @@ -483,11 +483,15 @@ Other minor additions
483
483
484
484
* Added new proof to ` Data.List.Relation.Binary.Subset.Setoid.Properties ` :
485
485
``` agda
486
+ xs⊆x∷xs : xs ⊆ x ∷ xs
487
+ ∷⁺ʳ : xs ⊆ ys → x ∷ xs ⊆ x ∷ ys
486
488
applyUpTo⁺ : m ≤ n → applyUpTo f m ⊆ applyUpTo f n
487
489
```
488
490
489
491
* Added new proof to ` Data.List.Relation.Binary.Subset.Propositional.Properties ` :
490
492
``` agda
493
+ xs⊆x∷xs : xs ⊆ x ∷ xs
494
+ ∷⁺ʳ : xs ⊆ ys → x ∷ xs ⊆ x ∷ ys
491
495
applyUpTo⁺ : m ≤ n → applyUpTo f m ⊆ applyUpTo f n
492
496
```
493
497
Original file line number Diff line number Diff line change @@ -133,6 +133,15 @@ map⁺ f xs⊆ys =
133
133
Prod.map₂ (Prod.map₁ xs⊆ys) ∘
134
134
_⟨$⟩_ (Inverse.from (map-∈↔ f))
135
135
136
+ ------------------------------------------------------------------------
137
+ -- ∷
138
+
139
+ xs⊆x∷xs : ∀ (xs : List A) x → xs ⊆ x ∷ xs
140
+ xs⊆x∷xs = Setoidₚ.xs⊆x∷xs (setoid _)
141
+
142
+ ∷⁺ʳ : ∀ x → xs ⊆ ys → x ∷ xs ⊆ x ∷ ys
143
+ ∷⁺ʳ = Setoidₚ.∷⁺ʳ (setoid _)
144
+
136
145
------------------------------------------------------------------------
137
146
-- _++_
138
147
Original file line number Diff line number Diff line change @@ -171,6 +171,19 @@ module _ (S : Setoid a ℓ) where
171
171
------------------------------------------------------------------------
172
172
-- Properties of list functions
173
173
------------------------------------------------------------------------
174
+ -- ∷
175
+
176
+ module _ (S : Setoid a ℓ) where
177
+
178
+ open Subset S
179
+
180
+ xs⊆x∷xs : ∀ xs x → xs ⊆ x ∷ xs
181
+ xs⊆x∷xs xs x = there
182
+
183
+ ∷⁺ʳ : ∀ {xs ys} x → xs ⊆ ys → x ∷ xs ⊆ x ∷ ys
184
+ ∷⁺ʳ x xs⊆ys (here p) = here p
185
+ ∷⁺ʳ x xs⊆ys (there p) = there (xs⊆ys p)
186
+
174
187
-- ++
175
188
176
189
module _ (S : Setoid a ℓ) where
You can’t perform that action at this time.
0 commit comments