Lemmas about List.Subset
, List.Sublist
, List.IsPrefix
, List.IsSuffix
, and List.IsInfix
. #
isPrefixOf #
@[simp]
isSuffixOf #
Subset #
List subset #
instance
List.instTransSubsetMem
{α : Type u_1}
:
Trans (fun (l₁ l₂ : List α) => l₂ ⊆ l₁) Membership.mem Membership.mem
Equations
- List.instTransSubsetMem = { trans := ⋯ }
Equations
- List.instTransSubset = { trans := ⋯ }
Sublist and isSublist #
Equations
- List.instTransSublist = { trans := ⋯ }
Equations
- List.instTransSublistSubset = { trans := ⋯ }
Equations
- List.instTransSubsetSublist = { trans := ⋯ }
instance
List.instTransSublistMem
{α : Type u_1}
:
Trans (fun (l₁ l₂ : List α) => l₂.Sublist l₁) Membership.mem Membership.mem
Equations
- List.instTransSublistMem = { trans := ⋯ }
Equations
- l₁.instDecidableSublistOfDecidableEq l₂ = decidable_of_iff (l₁.isSublist l₂ = true) ⋯
IsPrefix / IsSuffix / IsInfix #
Equations
- l₁.instDecidableIsPrefixOfDecidableEq l₂ = decidable_of_iff (l₁.isPrefixOf l₂ = true) ⋯
Equations
- l₁.instDecidableIsSuffixOfDecidableEq l₂ = decidable_of_iff (l₁.isSuffixOf l₂ = true) ⋯
Deprecations #
@[reducible, inline, deprecated List.sublist_flatten_iff (since := "2024-10-14")]
Equations
Instances For
@[reducible, inline, deprecated List.flatten_sublist_iff (since := "2024-10-14")]
Equations
Instances For
@[reducible, inline, deprecated List.infix_of_mem_flatten (since := "2024-10-14")]