Basic operations on List
. #
We define
- basic operations on
List
, - simp lemmas for applying the operations on
.nil
and.cons
arguments (in the cases where the right hand side is simple to state; otherwise these are deferred toInit.Data.List.Lemmas
), - the minimal lemmas which are required for setting up
Init.Data.Array.Basic
.
In Init.Data.List.Impl
we give tail-recursive versions of these operations
along with @[csimp]
lemmas,
In Init.Data.List.Lemmas
we develop the full API for these functions.
Recall that length
, get
, set
, foldl
, and concat
have already been defined in Init.Prelude
.
The operations are organized as follow:
- Equality:
beq
,isEqv
. - Lexicographic ordering:
lt
,le
, and instances. - Head and tail operators:
head
,head?
,headD?
,tail
,tail?
,tailD
. - Basic operations:
map
,filter
,filterMap
,foldr
,append
,flatten
,pure
,flatMap
,replicate
, andreverse
. - Additional functions defined in terms of these:
leftpad
,rightPad
, andreduceOption
. - Operations using indexes:
mapIdx
. - List membership:
isEmpty
,elem
,contains
,mem
(and the∈
notation), and decidability for predicates quantifying over membership in aList
. - Sublists:
take
,drop
,takeWhile
,dropWhile
,partition
,dropLast
,isPrefixOf
,isPrefixOf?
,isSuffixOf
,isSuffixOf?
,Subset
,Sublist
,rotateLeft
androtateRight
. - Manipulating elements:
replace
,modify
,insert
,insertIdx
,erase
,eraseP
,eraseIdx
. - Finding elements:
find?
,findSome?
,findIdx
,indexOf
,findIdx?
,indexOf?
,countP
,count
, andlookup
. - Logic:
any
,all
,or
, andand
. - Zippers:
zipWith
,zip
,zipWithAll
, andunzip
. - Ranges and enumeration:
range
,zipIdx
. - Minima and maxima:
min?
andmax?
. - Other functions:
intersperse
,intercalate
,eraseDups
,eraseReps
,span
,splitBy
,removeAll
(currently these functions are mostly only used in meta code, and do not have API suitable for verification).
Further operations are defined in Init.Data.List.BasicAux
(because they use Array
in their implementations), namely:
- Variant getters:
get!
,get?
,getD
,getLast
,getLast!
,getLast?
, andgetLastD
. - Head and tail:
head!
,tail!
. - Other operations on sublists:
partitionMap
,rotateLeft
, androtateRight
.
Preliminaries from Init.Prelude
#
length #
set #
foldl #
concat #
Equality #
Checks whether two lists have the same length and their elements are pairwise BEq
. Normally used
via the ==
operator.
Equations
Instances For
Equations
- Eq List.instBEq { beq := List.beq }
Instances For
Returns true
if as
and bs
have the same length and they are pairwise related by eqv
.
O(min |as| |bs|)
. Short-circuits at the first non-related pair of elements.
Examples:
[1, 2, 3].isEqv [2, 3, 4] (· < ·) = true
[1, 2, 3].isEqv [2, 2, 4] (· < ·) = false
[1, 2, 3].isEqv [2, 3] (· < ·) = false
Equations
Instances For
Lexicographic ordering #
Lexicographic ordering for lists with respect to an ordering of elements.
as
is lexicographically smaller than bs
if
as
is empty andbs
is non-empty, or- both
as
andbs
are non-empty, and the head ofas
is less than the head ofbs
according tor
, or - both
as
andbs
are non-empty, their heads are equal, and the tail ofas
is less than the tail ofbs
.
- nil
{α : Type u}
{r : α → α → Prop}
{a : α}
{l : List α}
: Lex r List.nil (List.cons a l)
[]
is the smallest element in the lexicographic order. - rel
{α : Type u}
{r : α → α → Prop}
{a₁ : α}
{l₁ : List α}
{a₂ : α}
{l₂ : List α}
(h : r a₁ a₂)
: Lex r (List.cons a₁ l₁) (List.cons a₂ l₂)
If the head of the first list is smaller than the head of the second, then the first list is lexicographically smaller than the second list.
- cons
{α : Type u}
{r : α → α → Prop}
{a : α}
{l₁ l₂ : List α}
(h : Lex r l₁ l₂)
: Lex r (List.cons a l₁) (List.cons a l₂)
If two lists have the same head, then their tails determine their lexicographic order. If the tail of the first list is lexicographically smaller than the tail of the second list, then the entire first list is lexicographically smaller than the entire second list.
Instances For
Instances For
Lexicographic ordering of lists with respect to an ordering on their elements.
as < bs
if
as
is empty andbs
is non-empty, or- both
as
andbs
are non-empty, and the head ofas
is less than the head ofbs
, or - both
as
andbs
are non-empty, their heads are equal, and the tail ofas
is less than the tail ofbs
.
Instances For
Equations
- Eq List.instLT { lt := List.lt }
Instances For
Decidability of lexicographic ordering.
Equations
- Eq (l₁.decidableLT l₂) (List.decidableLex (fun (x1 x2 : α) => LT.lt x1 x2) l₁ l₂)
Instances For
Decidability of lexicographic ordering.
Equations
Instances For
Non-strict ordering of lists with respect to a strict ordering of their elements.
as ≤ bs
if ¬ bs < as
.
This relation can be treated as a lexicographic order if the underlying LT α
instance is
well-behaved. In particular, it should be irreflexive, asymmetric, and antisymmetric. These
requirements are precisely formulated in List.cons_le_cons_iff
. If these hold, then as ≤ bs
if
and only if:
as
is empty, or- both
as
andbs
are non-empty, and the head ofas
is less than the head ofbs
, or - both
as
andbs
are non-empty, their heads are equal, and the tail ofas
is less than or equal to the tail ofbs
.
Instances For
Equations
- Eq List.instLE { le := List.le }
Instances For
Equations
- Eq (l₁.decidableLE l₂) (inferInstanceAs (Decidable (Not (LT.lt l₂ l₁))))
Instances For
Alternative getters #
getLast #
Returns the last element of a non-empty list.
Examples:
Equations
Instances For
getLast? #
Returns the last element in the list, or none
if the list is empty.
Alternatives include List.getLastD
, which takes a fallback value for empty lists, and
List.getLast!
, which panics on empty lists.
Examples:
["circle", "rectangle"].getLast? = some "rectangle"
["circle"].getLast? = some "circle"
([] : List String).getLast? = none
Equations
- Eq List.nil.getLast? Option.none
- Eq (List.cons a as).getLast? (Option.some ((List.cons a as).getLast ⋯))
Instances For
getLastD #
Returns the last element in the list, or fallback
if the list is empty.
Alternatives include List.getLast?
, which returns an Option
, and List.getLast!
, which panics
on empty lists.
Examples:
["circle", "rectangle"].getLastD "oval" = "rectangle"
["circle"].getLastD "oval" = "circle"
([] : List String).getLastD "oval" = "oval"
Equations
Instances For
Head and tail #
head #
head? #
Returns the first element in the list, if there is one. Returns none
if the list is empty.
Use List.headD
to provide a fallback value for empty lists, or List.head!
to panic on empty
lists.
Examples:
Equations
- Eq x✝.head? (List.getLast?.match_1 (fun (x : List α) => Option α) x✝ (fun (_ : Unit) => Option.none) fun (a : α) (tail : List α) => Option.some a)
Instances For
headD #
Returns the first element in the list if there is one, or fallback
if the list is empty.
Use List.head?
to return an Option
, and List.head!
to panic on empty lists.
Examples:
Instances For
tail #
tail? #
Drops the first element of a nonempty list, returning the tail. Returns none
when the argument is
empty.
Alternatives include List.tail
, which returns the empty list on failure, List.tailD
, which
returns an explicit fallback value, and List.tail!
, which panics on the empty list.
Examples:
["apple", "banana", "grape"].tail? = some ["banana", "grape"]
["apple"].tail? = some []
([] : List String).tail = none
Equations
- Eq x✝.tail? (List.getLast?.match_1 (fun (x : List α) => Option (List α)) x✝ (fun (_ : Unit) => Option.none) fun (head : α) (as : List α) => Option.some as)
Instances For
tailD #
Drops the first element of a nonempty list, returning the tail. Returns none
when the argument is
empty.
Alternatives include List.tail
, which returns the empty list on failure, List.tail?
, which
returns an Option
, and List.tail!
, which panics on the empty list.
Examples:
["apple", "banana", "grape"].tailD ["orange"] = ["banana", "grape"]
["apple"].tailD ["orange"] = []
[].tailD ["orange"] = ["orange"]
Equations
Instances For
Basic List
operations. #
We define the basic functional programming operations on List
:
map
, filter
, filterMap
, foldr
, append
, flatten
, pure
, bind
, replicate
, and reverse
.
map #
Applies a function to each element of the list, returning the resulting list of values.
O(|l|)
.
Examples:
[a, b, c].map f = [f a, f b, f c]
[].map Nat.succ = []
["one", "two", "three"].map (·.length) = [3, 3, 5]
["one", "two", "three"].map (·.reverse) = ["eno", "owt", "eerht"]
Equations
Instances For
filter #
Returns the list of elements in l
for which p
returns true
.
O(|l|)
.
Examples:
[1, 2, 5, 2, 7, 7].filter (· > 2) = [5, 7, 7]
[1, 2, 5, 2, 7, 7].filter (fun _ => false) = []
[1, 2, 5, 2, 7, 7].filter (fun _ => true) = [1, 2, 5, 2, 7, 7]
Equations
- Eq (List.filter p List.nil) List.nil
- Eq (List.filter p (List.cons a as)) (List.filter.match_1 (fun (x : Bool) => List α) (p a) (fun (_ : Unit) => List.cons a (List.filter p as)) fun (_ : Unit) => List.filter p as)
Instances For
filterMap #
Applies a function that returns an Option
to each element of a list, collecting the non-none
values.
O(|l|)
.
Example:
#eval [1, 2, 5, 2, 7, 7].filterMap fun x =>
if x > 2 then some (2 * x) else none
[10, 14, 14]
Equations
- Eq (List.filterMap f List.nil) List.nil
- Eq (List.filterMap f (List.cons a as)) (List.filterMap.match_1 (fun (x : Option β) => List β) (f a) (fun (_ : Unit) => List.filterMap f as) fun (b : β) => List.cons b (List.filterMap f as))
Instances For
foldr #
Folds a function over a list from the right, accumulating a value starting with init
. The
accumulated value is combined with the each element of the list in reverse order, using f
.
O(|l|)
. Replaced at runtime with List.foldrTR
.
Examples:
[a, b, c].foldr f init = f a (f b (f c init))
[1, 2, 3].foldr (toString · ++ ·) "" = "123"
[1, 2, 3].foldr (s!"({·} {·})") "!" = "(1 (2 (3 !)))"
Equations
- Eq (List.foldr f init List.nil) init
- Eq (List.foldr f init (List.cons a as)) (f a (List.foldr f init as))
Instances For
reverse #
Auxiliary for List.reverse
. List.reverseAux l r = l.reverse ++ r
, but it is defined directly.
Equations
- Eq (List.nil.reverseAux x✝) x✝
- Eq ((List.cons a l).reverseAux x✝) (l.reverseAux (List.cons a x✝))
Instances For
Reverses a list.
O(|as|)
.
Because of the “functional but in place” optimization implemented by Lean's compiler, this function does not allocate a new list when its reference to the input list is unshared: it simply walks the linked list and reverses all the node pointers.
Examples:
Equations
- Eq as.reverse (as.reverseAux List.nil)
Instances For
append #
Appends two lists. Normally used via the ++
operator.
Appending lists takes time proportional to the length of the first list: O(|xs|)
.
Examples:
[1, 2, 3] ++ [4, 5] = [1, 2, 3, 4, 5]
.[] ++ [4, 5] = [4, 5]
.[1, 2, 3] ++ [] = [1, 2, 3]
.
Instances For
Appends two lists. Normally used via the ++
operator.
Appending lists takes time proportional to the length of the first list: O(|xs|)
.
This is a tail-recursive version of List.append
.
Examples:
[1, 2, 3] ++ [4, 5] = [1, 2, 3, 4, 5]
.[] ++ [4, 5] = [4, 5]
.[1, 2, 3] ++ [] = [1, 2, 3]
.
Equations
- Eq (as.appendTR bs) (as.reverse.reverseAux bs)
Instances For
Equations
- Eq List.instAppend { append := List.append }
Instances For
flatten #
Concatenates a list of lists into a single list, preserving the order of the elements.
O(|flatten L|)
.
Examples:
[["a"], ["b", "c"]].flatten = ["a", "b", "c"]
[["a"], [], ["b", "c"], ["d", "e", "f"]].flatten = ["a", "b", "c", "d", "e", "f"]
Equations
Instances For
singleton #
Constructs a single-element list.
Examples:
List.singleton 5 = [5]
.List.singleton "green" = ["green"]
.List.singleton [1, 2, 3] = [[1, 2, 3]]
Equations
- Eq (List.singleton a) (List.cons a List.nil)
Instances For
flatMap #
Applies a function that returns a list to each element of a list, and concatenates the resulting lists.
Examples:
[2, 3, 2].flatMap List.range = [0, 1, 0, 1, 2, 0, 1]
["red", "blue"].flatMap String.toList = ['r', 'e', 'd', 'b', 'l', 'u', 'e']
Equations
- Eq (List.flatMap b as) (List.map b as).flatten
Instances For
Equations
Instances For
Equations
Instances For
replicate #
Creates a list that contains n
copies of a
.
List.replicate 5 "five" = ["five", "five", "five", "five", "five"]
List.replicate 0 "zero" = []
List.replicate 2 ' ' = [' ', ' ']
Equations
- Eq (List.replicate 0 x✝) List.nil
- Eq (List.replicate n.succ x✝) (List.cons x✝ (List.replicate n x✝))
Instances For
Additional functions #
leftpad and rightpad #
Pads l : List α
on the left with repeated occurrences of a : α
until it is of length n
. If l
already has at least n
elements, it is returned unmodified.
Examples:
[1, 2, 3].leftpad 5 0 = [0, 0, 1, 2, 3]
["red", "green", "blue"].leftpad 4 "blank" = ["blank", "red", "green", "blue"]
["red", "green", "blue"].leftpad 3 "blank" = ["red", "green", "blue"]
["red", "green", "blue"].leftpad 1 "blank" = ["red", "green", "blue"]
Equations
- Eq (List.leftpad n a l) (HAppend.hAppend (List.replicate (HSub.hSub n l.length) a) l)
Instances For
Pads l : List α
on the right with repeated occurrences of a : α
until it is of length n
. If
l
already has at least n
elements, it is returned unmodified.
Examples:
[1, 2, 3].rightpad 5 0 = [1, 2, 3, 0, 0]
["red", "green", "blue"].rightpad 4 "blank" = ["red", "green", "blue", "blank"]
["red", "green", "blue"].rightpad 3 "blank" = ["red", "green", "blue"]
["red", "green", "blue"].rightpad 1 "blank" = ["red", "green", "blue"]
Equations
- Eq (List.rightpad n a l) (HAppend.hAppend l (List.replicate (HSub.hSub n l.length) a))
Instances For
reduceOption #
Drop none
s from a list, and replace each remaining some a
with a
.
Equations
Instances For
List membership #
EmptyCollection #
Equations
- Eq List.instEmptyCollection { emptyCollection := List.nil }
Instances For
isEmpty #
elem #
Checks whether a
is an element of l
, using ==
to compare elements.
O(|l|)
. List.contains
is a synonym that takes the list before the element.
The preferred simp normal form is l.contains a
. When LawfulBEq α
is available,
l.contains a = true ↔ a ∈ l
and l.contains a = false ↔ a ∉ l
.
Example:
Equations
Instances For
contains #
Checks whether a
is an element of as
, using ==
to compare elements.
O(|as|)
. List.elem
is a synonym that takes the element before the list.
The preferred simp normal form is l.contains a
, and when LawfulBEq α
is available,
l.contains a = true ↔ a ∈ l
and l.contains a = false ↔ a ∉ l
.
Examples:
[1, 4, 2, 3, 3, 7].contains 3 = true
List.contains [1, 4, 2, 3, 3, 7] 5 = false
Instances For
Mem #
List membership, typically accessed via the ∈
operator.
a ∈ l
means that a
is an element of the list l
. Elements are compared according to Lean's
logical equality.
The related function List.elem
is a Boolean membership test that uses a BEq α
instance.
Examples:
a ∈ [x, y, z] ↔ a = x ∨ a = y ∨ a = z
- head
{α : Type u}
{a : α}
(as : List α)
: Mem a (cons a as)
The head of a list is a member:
a ∈ a :: as
. - tail
{α : Type u}
{a : α}
(b : α)
{as : List α}
: Mem a as → Mem a (cons b as)
A member of the tail of a list is a member of the list:
a ∈ l → a ∈ b :: l
.
Instances For
Equations
- Eq List.instMembership { mem := fun (l : List α) (a : α) => List.Mem a l }
Instances For
Equations
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Sublists #
take #
drop #
extract #
Returns the slice of l
from indices start
(inclusive) to stop
(exclusive).
Examples:
- [0, 1, 2, 3, 4, 5].extract 1 2 = [1]
- [0, 1, 2, 3, 4, 5].extract 2 2 = []
- [0, 1, 2, 3, 4, 5].extract 2 4 = [2, 3]
- [0, 1, 2, 3, 4, 5].extract 2 = [2, 3, 4, 5]
- [0, 1, 2, 3, 4, 5].extract (stop := 2) = [0, 1]
Instances For
takeWhile #
Returns the longest initial segment of xs
for which p
returns true.
O(|xs|)
.
Examples:
[7, 6, 4, 8].takeWhile (· > 5) = [7, 6]
[7, 6, 6, 5].takeWhile (· > 5) = [7, 6, 6]
[7, 6, 6, 8].takeWhile (· > 5) = [7, 6, 6, 8]
Equations
- Eq (List.takeWhile p List.nil) List.nil
- Eq (List.takeWhile p (List.cons a as)) (List.filter.match_1 (fun (x : Bool) => List α) (p a) (fun (_ : Unit) => List.cons a (List.takeWhile p as)) fun (_ : Unit) => List.nil)
Instances For
dropWhile #
Removes the longest prefix of a list for which p
returns true
.
Elements are removed from the list until one is encountered for which p
returns false
. This
element and the remainder of the list are returned.
O(|l|)
.
Examples:
[1, 3, 2, 4, 2, 7, 4].dropWhile (· < 4) = [4, 2, 7, 4]
[8, 3, 2, 4, 2, 7, 4].dropWhile (· < 4) = [8, 3, 2, 4, 2, 7, 4]
[8, 3, 2, 4, 2, 7, 4].dropWhile (· < 100) = []
Equations
- Eq (List.dropWhile p List.nil) List.nil
- Eq (List.dropWhile p (List.cons a as)) (List.filter.match_1 (fun (x : Bool) => List α) (p a) (fun (_ : Unit) => List.dropWhile p as) fun (_ : Unit) => List.cons a as)
Instances For
partition #
Returns a pair of lists that together contain all the elements of as
. The first list contains
those elements for which p
returns true
, and the second contains those for which p
returns
false
.
O(|l|)
. as.partition p
is equivalent to (as.filter p, as.filter (not ∘ p))
, but it is slightly
more efficient since it only has to do one pass over the list.
Examples:
[1, 2, 5, 2, 7, 7].partition (· > 2) = ([5, 7, 7], [1, 2, 2])
[1, 2, 5, 2, 7, 7].partition (fun _ => false) = ([], [1, 2, 5, 2, 7, 7])
[1, 2, 5, 2, 7, 7].partition (fun _ => true) = ([1, 2, 5, 2, 7, 7], [])
Equations
- Eq (List.partition p as) (List.partition.loop p as { fst := List.nil, snd := List.nil })
Instances For
Equations
- One or more equations did not get rendered due to their size.
- Eq (List.partition.loop p List.nil { fst := bs, snd := cs }) { fst := bs.reverse, snd := cs.reverse }
Instances For
dropLast #
Removes the last element of the list, if one exists.
Examples:
Equations
Instances For
Subset #
l₁ ⊆ l₂
means that every element of l₁
is also an element of l₂
, ignoring multiplicity.
Equations
- Eq (l₁.Subset l₂) (∀ ⦃a : α⦄, Membership.mem l₁ a → Membership.mem l₂ a)
Instances For
Equations
- Eq List.instHasSubset { Subset := List.Subset }
Instances For
Equations
- Eq (x✝¹.instDecidableRelSubsetOfDecidableEq x✝) (List.decidableBAll (Membership.mem x✝) x✝¹)
Instances For
Sublist and isSublist #
The first list is a non-contiguous sub-list of the second list. Typically written with the <+
operator.
In other words, l₁ <+ l₂
means that l₁
can be transformed into l₂
by repeatedly inserting new
elements.
- slnil
{α : Type u_1}
: nil.Sublist nil
The base case:
[]
is a sublist of[]
- cons
{α : Type u_1}
{l₁ l₂ : List α}
(a : α)
: l₁.Sublist l₂ → l₁.Sublist (List.cons a l₂)
If
l₁
is a subsequence ofl₂
, then it is also a subsequence ofa :: l₂
. - cons₂
{α : Type u_1}
{l₁ l₂ : List α}
(a : α)
: l₁.Sublist l₂ → (List.cons a l₁).Sublist (List.cons a l₂)
If
l₁
is a subsequence ofl₂
, thena :: l₁
is a subsequence ofa :: l₂
.
Instances For
The first list is a non-contiguous sub-list of the second list. Typically written with the <+
operator.
In other words, l₁ <+ l₂
means that l₁
can be transformed into l₂
by repeatedly inserting new
elements.
Equations
- Eq List.«term_<+_» (Lean.ParserDescr.trailingNode `List.«term_<+_» 50 50 (Lean.ParserDescr.binary `andthen (Lean.ParserDescr.symbol " <+ ") (Lean.ParserDescr.cat `term 51)))
Instances For
True if the first list is a potentially non-contiguous sub-sequence of the second list, comparing
elements with the ==
operator.
The relation List.Sublist
is a logical characterization of this property.
Examples:
Equations
Instances For
IsPrefix / isPrefixOf / isPrefixOf? #
The first list is a prefix of the second.
IsPrefix l₁ l₂
, written l₁ <+: l₂
, means that there exists some t : List α
such that l₂
has
the form l₁ ++ t
.
The function List.isPrefixOf
is a Boolean equivalent.
Conventions for notations in identifiers:
- The recommended spelling of
<+:
in identifiers isprefix
(notisPrefix
).
Instances For
The first list is a prefix of the second.
IsPrefix l₁ l₂
, written l₁ <+: l₂
, means that there exists some t : List α
such that l₂
has
the form l₁ ++ t
.
The function List.isPrefixOf
is a Boolean equivalent.
Conventions for notations in identifiers:
- The recommended spelling of
<+:
in identifiers isprefix
(notisPrefix
).
Equations
- Eq List.«term_<+:_» (Lean.ParserDescr.trailingNode `List.«term_<+:_» 50 50 (Lean.ParserDescr.binary `andthen (Lean.ParserDescr.symbol " <+: ") (Lean.ParserDescr.cat `term 51)))
Instances For
Checks whether the first list is a prefix of the second.
The relation List.IsPrefixOf
expresses this property with respect to logical equality.
Examples:
[1, 2].isPrefixOf [1, 2, 3] = true
[1, 2].isPrefixOf [1, 2] = true
[1, 2].isPrefixOf [1] = false
[1, 2].isPrefixOf [1, 1, 2, 3] = false
Equations
- Eq (List.nil.isPrefixOf x✝) Bool.true
- Eq (x✝.isPrefixOf List.nil) Bool.false
- Eq ((List.cons a as).isPrefixOf (List.cons b bs)) ((BEq.beq a b).and (as.isPrefixOf bs))
Instances For
If the first list is a prefix of the second, returns the result of dropping the prefix.
In other words, isPrefixOf? l₁ l₂
returns some t
when l₂ == l₁ ++ t
.
Examples:
[1, 2].isPrefixOf? [1, 2, 3] = some [3]
[1, 2].isPrefixOf? [1, 2] = some []
[1, 2].isPrefixOf? [1] = none
[1, 2].isPrefixOf? [1, 1, 2, 3] = none
Instances For
IsSuffix / isSuffixOf / isSuffixOf? #
Checks whether the first list is a suffix of the second.
The relation List.IsSuffixOf
expresses this property with respect to logical equality.
Examples:
[2, 3].isSuffixOf [1, 2, 3] = true
[2, 3].isSuffixOf [1, 2, 3, 4] = false
[2, 3].isSuffixOf [1, 2] = false
[2, 3].isSuffixOf [1, 1, 2, 3] = true
Equations
- Eq (l₁.isSuffixOf l₂) (l₁.reverse.isPrefixOf l₂.reverse)
Instances For
If the first list is a suffix of the second, returns the result of dropping the suffix from the second.
In other words, isSuffixOf? l₁ l₂
returns some t
when l₂ == t ++ l₁
.
Examples:
[2, 3].isSuffixOf? [1, 2, 3] = some [1]
[2, 3].isSuffixOf? [1, 2, 3, 4] = none
[2, 3].isSuffixOf? [1, 2] = none
[2, 3].isSuffixOf? [1, 1, 2, 3] = some [1, 1]
Equations
- Eq (l₁.isSuffixOf? l₂) (Option.map List.reverse (l₁.reverse.isPrefixOf? l₂.reverse))
Instances For
The first list is a suffix of the second.
IsSuffix l₁ l₂
, written l₁ <:+ l₂
, means that there exists some t : List α
such that l₂
has
the form t ++ l₁
.
The function List.isSuffixOf
is a Boolean equivalent.
Conventions for notations in identifiers:
- The recommended spelling of
<:+
in identifiers issuffix
(notisSuffix
).
Instances For
The first list is a suffix of the second.
IsSuffix l₁ l₂
, written l₁ <:+ l₂
, means that there exists some t : List α
such that l₂
has
the form t ++ l₁
.
The function List.isSuffixOf
is a Boolean equivalent.
Conventions for notations in identifiers:
- The recommended spelling of
<:+
in identifiers issuffix
(notisSuffix
).
Equations
- Eq List.«term_<:+_» (Lean.ParserDescr.trailingNode `List.«term_<:+_» 50 50 (Lean.ParserDescr.binary `andthen (Lean.ParserDescr.symbol " <:+ ") (Lean.ParserDescr.cat `term 51)))
Instances For
IsInfix #
The first list is a contiguous sub-list of the second list. Typically written with the <:+:
operator.
In other words, l₁ <:+: l₂
means that there exist lists s : List α
and t : List α
such that
l₂
has the form s ++ l₁ ++ t
.
Conventions for notations in identifiers:
- The recommended spelling of
<:+:
in identifiers isinfix
(notisInfix
).
Equations
- Eq (l₁.IsInfix l₂) (Exists fun (s : List α) => Exists fun (t : List α) => Eq (HAppend.hAppend (HAppend.hAppend s l₁) t) l₂)
Instances For
The first list is a contiguous sub-list of the second list. Typically written with the <:+:
operator.
In other words, l₁ <:+: l₂
means that there exist lists s : List α
and t : List α
such that
l₂
has the form s ++ l₁ ++ t
.
Conventions for notations in identifiers:
- The recommended spelling of
<:+:
in identifiers isinfix
(notisInfix
).
Equations
- Eq List.«term_<:+:_» (Lean.ParserDescr.trailingNode `List.«term_<:+:_» 50 50 (Lean.ParserDescr.binary `andthen (Lean.ParserDescr.symbol " <:+: ") (Lean.ParserDescr.cat `term 51)))
Instances For
splitAt #
Splits a list at an index, resulting in the first n
elements of l
paired with the remaining
elements.
If n
is greater than the length of l
, then the resulting pair consists of l
and the empty
list. List.splitAt
is equivalent to a combination of List.take
and List.drop
, but it is more
efficient.
Examples:
["red", "green", "blue"].splitAt 2 = (["red", "green"], ["blue"])
["red", "green", "blue"].splitAt 3 = (["red", "green", "blue], [])
["red", "green", "blue"].splitAt 4 = (["red", "green", "blue], [])
Equations
- Eq (List.splitAt n l) (List.splitAt.go l l n List.nil)
Instances For
Auxiliary for splitAt
:
splitAt.go l xs n acc = (acc.reverse ++ take n xs, drop n xs)
if n < xs.length
,
and (l, [])
otherwise.
Equations
- Eq (List.splitAt.go l List.nil x✝¹ x✝) { fst := l, snd := List.nil }
- Eq (List.splitAt.go l (List.cons x_3 xs) n.succ x✝) (List.splitAt.go l xs n (List.cons x_3 x✝))
- Eq (List.splitAt.go l x✝² x✝¹ x✝) { fst := x✝.reverse, snd := x✝² }
Instances For
rotateLeft #
Rotates the elements of xs
to the left, moving i % xs.length
elements from the start of the list
to the end.
O(|xs|)
.
Examples:
[1, 2, 3, 4, 5].rotateLeft 3 = [4, 5, 1, 2, 3]
[1, 2, 3, 4, 5].rotateLeft 5 = [1, 2, 3, 4, 5]
[1, 2, 3, 4, 5].rotateLeft 1 = [2, 3, 4, 5, 1]
Equations
- Eq (xs.rotateLeft i) (ite (LE.le xs.length 1) xs (let i := HMod.hMod i xs.length; let ys := List.take i xs; let zs := List.drop i xs; HAppend.hAppend zs ys))
Instances For
rotateRight #
Rotates the elements of xs
to the right, moving i % xs.length
elements from the end of the list
to the start.
After rotation, the element at xs[n]
is at index (i + n) % l.length
. O(|xs|)
.
Examples:
[1, 2, 3, 4, 5].rotateRight 3 = [3, 4, 5, 1, 2]
[1, 2, 3, 4, 5].rotateRight 5 = [1, 2, 3, 4, 5]
[1, 2, 3, 4, 5].rotateRight 1 = [5, 1, 2, 3, 4]
Equations
Instances For
Pairwise, Nodup #
Each element of a list is related to all later elements of the list by R
.
Pairwise R l
means that all the elements of l
with earlier indexes are R
-related to all the
elements with later indexes.
For example, Pairwise (· ≠ ·) l
asserts that l
has no duplicates, and if Pairwise (· < ·) l
asserts that l
is (strictly) sorted.
Examples:
Pairwise (· < ·) [1, 2, 3] ↔ (1 < 2 ∧ 1 < 3) ∧ 2 < 3
Pairwise (· = ·) [1, 2, 3] = False
Pairwise (· ≠ ·) [1, 2, 3] = True
- nil
{α : Type u}
{R : α → α → Prop}
: Pairwise R List.nil
All elements of the empty list are vacuously pairwise related.
- cons {α : Type u} {R : α → α → Prop} {a : α} {l : List α} : (∀ (a' : α), Membership.mem l a' → R a a') → Pairwise R l → Pairwise R (List.cons a l)
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
The list has no duplicates: it contains every element at most once.
It is defined as Pairwise (· ≠ ·)
: each element is unequal to all other elements.
Equations
- Eq List.Nodup (List.Pairwise fun (x1 x2 : α) => Ne x1 x2)
Instances For
Instances For
Manipulating elements #
replace #
modify #
Replaces the n
th tail of l
with the result of applying f
to it. Returns the input without
using f
if the index is larger than the length of the List.
Examples:
["circle", "square", "triangle"].modifyTailIdx 1 List.reverse
["circle", "triangle", "square"]
["circle", "square", "triangle"].modifyTailIdx 1 (fun xs => xs ++ xs)
["circle", "square", "triangle", "square", "triangle"]
["circle", "square", "triangle"].modifyTailIdx 2 (fun xs => xs ++ xs)
["circle", "square", "triangle", "triangle"]
["circle", "square", "triangle"].modifyTailIdx 5 (fun xs => xs ++ xs)
["circle", "square", "triangle"]
Equations
- Eq (l.modifyTailIdx i f) (List.modifyTailIdx.go f i l)
Instances For
Replace the head of the list with the result of applying f
to it. Returns the empty list if the
list is empty.
Examples:
[1, 2, 3].modifyHead (· * 10) = [10, 2, 3]
[].modifyHead (· * 10) = []
Equations
- Eq (List.modifyHead f List.nil) List.nil
- Eq (List.modifyHead f (List.cons a as)) (List.cons (f a) as)
Instances For
Replaces the element at the given index, if it exists, with the result of applying f
to it. If the
index is invalid, the list is returned unmodified.
Examples:
[1, 2, 3].modify 0 (· * 10) = [10, 2, 3]
[1, 2, 3].modify 2 (· * 10) = [1, 2, 30]
[1, 2, 3].modify 3 (· * 10) = [1, 2, 3]
Equations
- Eq (l.modify i f) (l.modifyTailIdx i (List.modifyHead f))
Instances For
insert #
Inserts an element into a list without duplication.
If the element is present in the list, the list is returned unmodified. Otherwise, the new element is inserted at the head of the list.
Examples:
Instances For
Inserts an element into a list at the specified index. If the index is greater than the length of the list, then the list is returned unmodified.
In other words, the new element is inserted into the list l
after the first i
elements of l
.
Examples:
["tues", "thur", "sat"].insertIdx 1 "wed" = ["tues", "wed", "thur", "sat"]
["tues", "thur", "sat"].insertIdx 2 "wed" = ["tues", "thur", "wed", "sat"]
["tues", "thur", "sat"].insertIdx 3 "wed" = ["tues", "thur", "sat", "wed"]
["tues", "thur", "sat"].insertIdx 4 "wed" = ["tues", "thur", "sat"]
Equations
- Eq (xs.insertIdx i a) (xs.modifyTailIdx i (List.cons a))
Instances For
erase #
Removes the first occurrence of a
from l
. If a
does not occur in l
, the list is returned
unmodified.
O(|l|)
.
Examples:
Equations
Instances For
Removes the first element of a list for which p
returns true
. If no element satisfies p
, then
the list is returned unchanged.
Examples:
[2, 1, 2, 1, 3, 4].eraseP (· < 2) = [2, 2, 1, 3, 4]
[2, 1, 2, 1, 3, 4].eraseP (· > 2) = [2, 1, 2, 1, 4]
[2, 1, 2, 1, 3, 4].eraseP (· > 8) = [2, 1, 2, 1, 3, 4]
Equations
- Eq (List.eraseP p List.nil) List.nil
- Eq (List.eraseP p (List.cons a as)) (bif p a then as else List.cons a (List.eraseP p as))
Instances For
eraseIdx #
Finding elements
find? #
Returns the first element of the list for which the predicate p
returns true
, or none
if no
such element is found.
O(|l|)
.
Examples:
Equations
- Eq (List.find? p List.nil) Option.none
- Eq (List.find? p (List.cons a as)) (List.filter.match_1 (fun (x : Bool) => Option α) (p a) (fun (_ : Unit) => Option.some a) fun (_ : Unit) => List.find? p as)
Instances For
findSome? #
Returns the first non-none
result of applying f
to each element of the list in order. Returns
none
if f
returns none
for all elements of the list.
O(|l|)
.
Examples:
[7, 6, 5, 8, 1, 2, 6].findSome? (fun x => if x < 5 then some (10 * x) else none) = some 10
[7, 6, 5, 8, 1, 2, 6].findSome? (fun x => if x < 1 then some (10 * x) else none) = none
Equations
- Eq (List.findSome? f List.nil) Option.none
- Eq (List.findSome? f (List.cons a as)) (List.findSome?.match_1 (fun (x : Option β) => Option β) (f a) (fun (b : β) => Option.some b) fun (_ : Unit) => List.findSome? f as)
Instances For
findIdx #
Returns the index of the first element for which p
returns true
, or the length of the list if
there is no such element.
Examples:
Equations
- Eq (List.findIdx p l) (List.findIdx.go p l 0)
Instances For
Auxiliary for findIdx
: findIdx.go p l n = findIdx p l + n
Equations
- Eq (List.findIdx.go p List.nil x✝) x✝
- Eq (List.findIdx.go p (List.cons a l) x✝) (bif p a then x✝ else List.findIdx.go p l (HAdd.hAdd x✝ 1))
Instances For
idxOf #
Returns the index of the first element equal to a
, or the length of the list if no element is
equal to a
.
Examples:
["carrot", "potato", "broccoli"].idxOf "carrot" = 0
["carrot", "potato", "broccoli"].idxOf "broccoli" = 2
["carrot", "potato", "broccoli"].idxOf "tomato" = 3
["carrot", "potato", "broccoli"].idxOf "anything else" = 3
Equations
- Eq (List.idxOf a) (List.findIdx fun (x : α) => BEq.beq x a)
Instances For
Returns the index of the first element equal to a
, or the length of the list otherwise.
Equations
Instances For
findIdx? #
Returns the index of the first element for which p
returns true
, or none
if there is no such
element.
Examples:
Equations
- Eq (List.findIdx? p l) (List.findIdx?.go p l 0)
Instances For
Equations
- Eq (List.findIdx?.go p List.nil x✝) Option.none
- Eq (List.findIdx?.go p (List.cons a l) x✝) (ite (Eq (p a) Bool.true) (Option.some x✝) (List.findIdx?.go p l (HAdd.hAdd x✝ 1)))
Instances For
idxOf? #
Returns the index of the first element equal to a
, or none
if no element is equal to a
.
Examples:
["carrot", "potato", "broccoli"].idxOf? "carrot" = some 0
["carrot", "potato", "broccoli"].idxOf? "broccoli" = some 2
["carrot", "potato", "broccoli"].idxOf? "tomato" = none
["carrot", "potato", "broccoli"].idxOf? "anything else" = none
Equations
- Eq (List.idxOf? a) (List.findIdx? fun (x : α) => BEq.beq x a)
Instances For
Return the index of the first occurrence of a
in the list.
Equations
Instances For
findFinIdx? #
Returns the index of the first element for which p
returns true
, or none
if there is no such
element. The index is returned as a Fin
, which guarantees that it is in bounds.
Examples:
[7, 6, 5, 8, 1, 2, 6].findFinIdx? (· < 5) = some (4 : Fin 7)
[7, 6, 5, 8, 1, 2, 6].findFinIdx? (· < 1) = none
Equations
- Eq (List.findFinIdx? p l) (List.findFinIdx?.go p l l 0 ⋯)
Instances For
Equations
- Eq (List.findFinIdx?.go p l List.nil x x_1) Option.none
- Eq (List.findFinIdx?.go p l (List.cons a l_1) x x_1) (ite (Eq (p a) Bool.true) (Option.some ⟨x, ⋯⟩) (List.findFinIdx?.go p l l_1 (HAdd.hAdd x 1) ⋯))
Instances For
finIdxOf? #
Returns the index of the first element equal to a
, or the length of the list if no element is
equal to a
. The index is returned as a Fin
, which guarantees that it is in bounds.
Examples:
["carrot", "potato", "broccoli"].finIdxOf? "carrot" = some 0
["carrot", "potato", "broccoli"].finIdxOf? "broccoli" = some 2
["carrot", "potato", "broccoli"].finIdxOf? "tomato" = none
["carrot", "potato", "broccoli"].finIdxOf? "anything else" = none
Equations
- Eq (List.finIdxOf? a) (List.findFinIdx? fun (x : α) => BEq.beq x a)
Instances For
countP #
Counts the number of elements in the list l
that satisfy the Boolean predicate p
.
Examples:
[1, 2, 3, 4, 5].countP (· % 2 == 0) = 2
[1, 2, 3, 4, 5].countP (· < 5) = 4
[1, 2, 3, 4, 5].countP (· > 5) = 0
Equations
- Eq (List.countP p l) (List.countP.go p l 0)
Instances For
Auxiliary for countP
: countP.go p l acc = countP p l + acc
.
Equations
- Eq (List.countP.go p List.nil x✝) x✝
- Eq (List.countP.go p (List.cons a l) x✝) (bif p a then List.countP.go p l (HAdd.hAdd x✝ 1) else List.countP.go p l x✝)
Instances For
count #
Counts the number of times an element occurs in a list.
Examples:
Equations
- Eq (List.count a) (List.countP fun (x : α) => BEq.beq x a)
Instances For
lookup #
Treats the list as an association list that maps keys to values, returning the first value whose key is equal to the specified key.
O(|l|)
.
Examples:
[(1, "one"), (3, "three"), (3, "other")].lookup 3 = some "three"
[(1, "one"), (3, "three"), (3, "other")].lookup 2 = none
Equations
- One or more equations did not get rendered due to their size.
Instances For
Permutations #
Perm #
Two lists are permutations of each other if they contain the same elements, each occurring the same number of times but not necessarily in the same order.
One list can be proven to be a permutation of another by showing how to transform one into the other by repeatedly swapping adjacent elements.
List.isPerm
is a Boolean equivalent of this relation.
- nil
{α : Type u}
: List.nil.Perm List.nil
The empty list is a permutation of the empty list:
[] ~ []
. - cons
{α : Type u}
(x : α)
{l₁ l₂ : List α}
: l₁.Perm l₂ → (List.cons x l₁).Perm (List.cons x l₂)
If one list is a permutation of the other, adding the same element as the head of each yields lists that are permutations of each other:
l₁ ~ l₂ → x::l₁ ~ x::l₂
. - swap
{α : Type u}
(x y : α)
(l : List α)
: (List.cons y (List.cons x l)).Perm (List.cons x (List.cons y l))
If two lists are identical except for having their first two elements swapped, then they are permutations of each other:
x::y::l ~ y::x::l
. - trans
{α : Type u}
{l₁ l₂ l₃ : List α}
: l₁.Perm l₂ → l₂.Perm l₃ → l₁.Perm l₃
Permutation is transitive:
l₁ ~ l₂ → l₂ ~ l₃ → l₁ ~ l₃
.
Instances For
Two lists are permutations of each other if they contain the same elements, each occurring the same number of times but not necessarily in the same order.
One list can be proven to be a permutation of another by showing how to transform one into the other by repeatedly swapping adjacent elements.
List.isPerm
is a Boolean equivalent of this relation.
Equations
- Eq List.«term_~_» (Lean.ParserDescr.trailingNode `List.«term_~_» 50 50 (Lean.ParserDescr.binary `andthen (Lean.ParserDescr.symbol " ~ ") (Lean.ParserDescr.cat `term 51)))
Instances For
isPerm #
Returns true
if l₁
and l₂
are permutations of each other. O(|l₁| * |l₂|)
.
The relation List.Perm
is a logical characterization of permutations. When the BEq α
instance
corresponds to DecidableEq α
, isPerm l₁ l₂ ↔ l₁ ~ l₂
(use the theorem isPerm_iff
).
Equations
Instances For
Logical operations #
any #
all #
or #
and #
Zippers #
zipWith #
Applies a function to the corresponding elements of two lists, stopping at the end of the shorter list.
O(min |xs| |ys|)
.
Examples:
[1, 2].zipWith (· + ·) [5, 6] = [6, 8]
[1, 2, 3].zipWith (· + ·) [5, 6, 10] = [6, 8, 13]
[].zipWith (· + ·) [5, 6] = []
[x₁, x₂, x₃].zipWith f [y₁, y₂, y₃, y₄] = [f x₁ y₁, f x₂ y₂, f x₃ y₃]
Equations
- Eq (List.zipWith f (List.cons x_2 xs) (List.cons y ys)) (List.cons (f x_2 y) (List.zipWith f xs ys))
- Eq (List.zipWith f x✝¹ x✝) List.nil
Instances For
zip #
Combines two lists into a list of pairs in which the first and second components are the corresponding elements of each list. The resulting list is the length of the shorter of the input lists.
O(min |xs| |ys|)
.
Examples:
["Mon", "Tue", "Wed"].zip [1, 2, 3] = [("Mon", 1), ("Tue", 2), ("Wed", 3)]
["Mon", "Tue", "Wed"].zip [1, 2] = [("Mon", 1), ("Tue", 2)]
[x₁, x₂, x₃].zip [y₁, y₂, y₃, y₄] = [(x₁, y₁), (x₂, y₂), (x₃, y₃)]
Equations
Instances For
zipWithAll #
Applies a function to the corresponding elements of both lists, stopping when there are no more
elements in either list. If one list is shorter than the other, the function is passed none
for
the missing elements.
Examples:
[1, 6].zipWithAll min [5, 2] = [some 1, some 2]
[1, 2, 3].zipWithAll Prod.mk [5, 6] = [(some 1, some 5), (some 2, some 6), (some 3, none)]
[x₁, x₂].zipWithAll f [y] = [f (some x₁) (some y), f (some x₂) none]
Instances For
unzip #
Separates a list of pairs into two lists that contain the respective first and second components.
O(|l|)
.
Examples:
[("Monday", 1), ("Tuesday", 2)].unzip = (["Monday", "Tuesday"], [1, 2])
[(x₁, y₁), (x₂, y₂), (x₃, y₃)].unzip = ([x₁, x₂, x₃], [y₁, y₂, y₃])
([] : List (Nat × String)).unzip = (([], []) : List Nat × List String)
Equations
- One or more equations did not get rendered due to their size.
Instances For
Ranges and enumeration #
range #
Returns a list of the numbers from 0
to n
exclusive, in increasing order.
O(n)
.
Examples:
Equations
- Eq (List.range n) (List.range.loop n List.nil)
Instances For
range' #
Returns a list of the numbers with the given length len
, starting at start
and increasing by
step
at each element.
In other words, List.range' start len step
is [start, start+step, ..., start+(len-1)*step]
.
Examples:
List.range' 0 3 (step := 1) = [0, 1, 2]
List.range' 0 3 (step := 2) = [0, 2, 4]
List.range' 0 4 (step := 2) = [0, 2, 4, 6]
List.range' 3 4 (step := 2) = [3, 5, 7, 9]
Equations
- Eq (List.range' x✝¹ 0 x✝) List.nil
- Eq (List.range' x✝¹ n.succ x✝) (List.cons x✝¹ (List.range' (HAdd.hAdd x✝¹ x✝) n x✝))
Instances For
iota #
zipIdx #
Pairs each element of a list with its index, optionally starting from an index other than 0
.
O(|l|)
.
Examples:
Equations
Instances For
enumFrom #
O(|l|)
. enumFrom n l
is like enum
but it allows you to specify the initial index.
enumFrom 5 [a, b, c] = [(5, a), (6, b), (7, c)]
Equations
- Eq (List.enumFrom x✝ List.nil) List.nil
- Eq (List.enumFrom x✝ (List.cons x_2 xs)) (List.cons { fst := x✝, snd := x_2 } (List.enumFrom (HAdd.hAdd x✝ 1) xs))
Instances For
enum #
O(|l|)
. enum l
pairs up each element with its index in the list.
enum [a, b, c] = [(0, a), (1, b), (2, c)]
Equations
- Eq List.enum (List.enumFrom 0)
Instances For
Minima and maxima #
min? #
Returns the smallest element of the list if it is not empty, or none
if it is empty.
Examples:
Equations
- Eq List.nil.min? Option.none
- Eq (List.cons a as).min? (Option.some (List.foldl Min.min a as))
Instances For
Returns the smallest element of the list if it is not empty, or none
if it is empty.
Examples:
Equations
Instances For
max? #
Returns the largest element of the list if it is not empty, or none
if it is empty.
Examples:
Equations
- Eq List.nil.max? Option.none
- Eq (List.cons a as).max? (Option.some (List.foldl Max.max a as))
Instances For
Returns the largest element of the list if it is not empty, or none
if it is empty.
Examples:
Equations
Instances For
Other list operations #
The functions are currently mostly used in meta code, and do not have sufficient API developed for verification work.
intersperse #
Alternates the elements of l
with sep
.
O(|l|)
.
List.intercalate
is a similar function that alternates a separator list with elements of a list of
lists.
Examples:
List.intersperse "then" [] = []
List.intersperse "then" ["walk"] = ["walk"]
List.intersperse "then" ["walk", "run"] = ["walk", "then", "run"]
List.intersperse "then" ["walk", "run", "rest"] = ["walk", "then", "run", "then", "rest"]
Equations
- Eq (List.intersperse sep List.nil) List.nil
- Eq (List.intersperse sep (List.cons head List.nil)) (List.cons head List.nil)
- Eq (List.intersperse sep (List.cons a as)) (List.cons a (List.cons sep (List.intersperse sep as)))
Instances For
intercalate #
Alternates the lists in xs
with the separator sep
, appending them. The resulting list is
flattened.
O(|xs|)
.
List.intersperse
is a similar function that alternates a separator element with the elements of a
list.
Examples:
List.intercalate sep [] = []
List.intercalate sep [a] = a
List.intercalate sep [a, b] = a ++ sep ++ b
List.intercalate sep [a, b, c] = a ++ sep ++ b ++ sep ++ c
Equations
- Eq (sep.intercalate xs) (List.intersperse sep xs).flatten
Instances For
eraseDups #
eraseReps #
Erases repeated elements, keeping the first element of each run.
O(|l|)
.
Example:
[1, 3, 2, 2, 2, 3, 3, 5].eraseReps = [1, 3, 2, 3, 5]
Equations
- Eq x✝.eraseReps (List.getLast?.match_1 (fun (x : List α) => List α) x✝ (fun (_ : Unit) => List.nil) fun (a : α) (as : List α) => List.eraseReps.loop a as List.nil)
Instances For
span #
Splits a list into the the longest initial segment for which p
returns true
, paired with the
remainder of the list.
O(|l|)
.
Examples:
[6, 8, 9, 5, 2, 9].span (· > 5) = ([6, 8, 9], [5, 2, 9])
[6, 8, 9, 5, 2, 9].span (· > 10) = ([], [6, 8, 9, 5, 2, 9])
[6, 8, 9, 5, 2, 9].span (· > 0) = ([6, 8, 9, 5, 2, 9], [])
Equations
- Eq (List.span p as) (List.span.loop p as List.nil)
Instances For
splitBy #
Splits a list into the longest segments in which each pair of adjacent elements are related by R
.
O(|l|)
.
Examples:
[1, 1, 2, 2, 2, 3, 2].splitBy (· == ·) = [[1, 1], [2, 2, 2], [3], [2]]
[1, 2, 5, 4, 5, 1, 4].splitBy (· < ·) = [[1, 2, 5], [4, 5], [1, 4]]
[1, 2, 5, 4, 5, 1, 4].splitBy (fun _ _ => true) = [[1, 2, 5, 4, 5, 1, 4]]
[1, 2, 5, 4, 5, 1, 4].splitBy (fun _ _ => false) = [[1], [2], [5], [4], [5], [1], [4]]
Equations
- Eq (List.splitBy R x✝) (List.getLast?.match_1 (fun (x : List α) => List (List α)) x✝ (fun (_ : Unit) => List.nil) fun (a : α) (as : List α) => List.splitBy.loop R as a List.nil List.nil)
Instances For
The arguments of splitBy.loop l b g gs
represent the following:
l : List α
are the elements which we still need to split.b : α
is the previous element for which a comparison was performed.r : List α
is the group currently being assembled, in reverse order.acc : List (List α)
is all of the groups that have been completed, in reverse order.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Splits a list into the longest segments in which each pair of adjacent elements are related by R
.
O(|l|)
.
Examples:
[1, 1, 2, 2, 2, 3, 2].splitBy (· == ·) = [[1, 1], [2, 2, 2], [3], [2]]
[1, 2, 5, 4, 5, 1, 4].splitBy (· < ·) = [[1, 2, 5], [4, 5], [1, 4]]
[1, 2, 5, 4, 5, 1, 4].splitBy (fun _ _ => true) = [[1, 2, 5, 4, 5, 1, 4]]
[1, 2, 5, 4, 5, 1, 4].splitBy (fun _ _ => false) = [[1], [2], [5], [4], [5], [1], [4]]
Equations
Instances For
removeAll #
Removes all elements of xs
that are present in ys
.
O(|xs| * |ys|)
.
Examples:
[1, 1, 5, 1, 2, 4, 5].removeAll [1, 2, 2] = [5, 4, 5]
[1, 2, 3, 2].removeAll [] = [1, 2, 3, 2]
[1, 2, 3, 2].removeAll [3] = [1, 2, 2]
Equations
- Eq (xs.removeAll ys) (List.filter (fun (x : α) => (List.elem x ys).not) xs)
Instances For
Runtime re-implementations using @[csimp]
#
More of these re-implementations are provided in Init/Data/List/Impl.lean
.
They can not be here, because the remaining ones required Array
for their implementation.
This leaves a dangerous situation: if you import this file, but not Init/Data/List/Impl.lean
,
then at runtime you will get non tail-recursive versions.
length #
map #
Applies a function to each element of the list, returning the resulting list of values.
O(|l|)
. This is the tail-recursive variant of List.map
, used in runtime code.
Examples:
[a, b, c].mapTR f = [f a, f b, f c]
[].mapTR Nat.succ = []
["one", "two", "three"].mapTR (·.length) = [3, 3, 5]
["one", "two", "three"].mapTR (·.reverse) = ["eno", "owt", "eerht"]
Equations
- Eq (List.mapTR f as) (List.mapTR.loop f as List.nil)
Instances For
Equations
- Eq (List.mapTR.loop f List.nil x✝) x✝.reverse
- Eq (List.mapTR.loop f (List.cons a as) x✝) (List.mapTR.loop f as (List.cons (f a) x✝))
Instances For
filter #
Returns the list of elements in l
for which p
returns true
.
O(|l|)
. This is a tail-recursive version of List.filter
, used at runtime.
Examples:
[1, 2, 5, 2, 7, 7].filterTR (· > 2) = [5, 7, 7]
[1, 2, 5, 2, 7, 7].filterTR (fun _ => false) = []
[1, 2, 5, 2, 7, 7].filterTR (fun _ => true) = * [1, 2, 5, 2, 7, 7]
Equations
- Eq (List.filterTR p as) (List.filterTR.loop p as List.nil)
Instances For
replicate #
Creates a list that contains n
copies of a
.
This is a tail-recursive version of List.replicate
.
List.replicateTR 5 "five" = ["five", "five", "five", "five", "five"]
List.replicateTR 0 "zero" = []
List.replicateTR 2 ' ' = [' ', ' ']
Equations
- Eq (List.replicateTR n a) (List.replicateTR.loop a n List.nil)
Instances For
Equations
- Eq (List.replicateTR.loop a 0 x✝) x✝
- Eq (List.replicateTR.loop a n.succ x✝) (List.replicateTR.loop a n (List.cons a x✝))
Instances For
Additional functions #
leftpad #
Pads l : List α
on the left with repeated occurrences of a : α
until it is of length n
. If l
already has at least n
elements, it is returned unmodified.
This is a tail-recursive version of List.leftpad
, used at runtime.
Examples:
[1, 2, 3].leftPadTR 5 0 = [0, 0, 1, 2, 3]
["red", "green", "blue"].leftPadTR 4 "blank" = ["blank", "red", "green", "blue"]
["red", "green", "blue"].leftPadTR 3 "blank" = ["red", "green", "blue"]
["red", "green", "blue"].leftPadTR 1 "blank" = ["red", "green", "blue"]
Equations
- Eq (List.leftpadTR n a l) (List.replicateTR.loop a (HSub.hSub n l.length) l)
Instances For
Zippers #
unzip #
Separates a list of pairs into two lists that contain the respective first and second components.
O(|l|)
. This is a tail-recursive version of List.unzip
that's used at runtime.
Examples:
[("Monday", 1), ("Tuesday", 2)].unzipTR = (["Monday", "Tuesday"], [1, 2])
[(x₁, y₁), (x₂, y₂), (x₃, y₃)].unzipTR = ([x₁, x₂, x₃], [y₁, y₂, y₃])
([] : List (Nat × String)).unzipTR = (([], []) : List Nat × List String)
Equations
- One or more equations did not get rendered due to their size.
Instances For
Ranges and enumeration #
range' #
Returns a list of the numbers with the given length len
, starting at start
and increasing by
step
at each element.
In other words, List.range'TR start len step
is [start, start+step, ..., start+(len-1)*step]
.
This is a tail-recursive version of List.range'
.
Examples:
List.range'TR 0 3 (step := 1) = [0, 1, 2]
List.range'TR 0 3 (step := 2) = [0, 2, 4]
List.range'TR 0 4 (step := 2) = [0, 2, 4, 6]
List.range'TR 3 4 (step := 2) = [3, 5, 7, 9]
Equations
- Eq (List.range'TR s n step) (List.range'TR.go step n (HAdd.hAdd s (HMul.hMul step n)) List.nil)
Instances For
Auxiliary for range'TR
: range'TR.go n e = [e-n, ..., e-1] ++ acc
.
Equations
- Eq (List.range'TR.go step 0 x✝¹ x✝) x✝
- Eq (List.range'TR.go step n.succ x✝¹ x✝) (List.range'TR.go step n (HSub.hSub x✝¹ step) (List.cons (HSub.hSub x✝¹ step) x✝))
Instances For
iota #
Tail-recursive version of List.iota
.
Equations
- Eq (List.iotaTR n) (List.iotaTR.go n List.nil)
Instances For
Equations
- Eq (List.iotaTR.go 0 x✝) x✝.reverse
- Eq (List.iotaTR.go n.succ x✝) (List.iotaTR.go n (List.cons n.succ x✝))
Instances For
Other list operations #
intersperse #
Alternates the elements of l
with sep
.
O(|l|)
.
This is a tail-recursive version of List.intersperse
, used at runtime.
Examples:
List.intersperseTR "then" [] = []
List.intersperseTR "then" ["walk"] = ["walk"]
List.intersperseTR "then" ["walk", "run"] = ["walk", "then", "run"]
List.intersperseTR "then" ["walk", "run", "rest"] = ["walk", "then", "run", "then", "rest"]
Equations
- Eq (List.intersperseTR sep List.nil) List.nil
- Eq (List.intersperseTR sep (List.cons x_1 List.nil)) (List.cons x_1 List.nil)
- Eq (List.intersperseTR sep (List.cons x_1 (List.cons y xs))) (List.cons x_1 (List.cons sep (List.cons y (List.foldr (fun (a : α) (r : List α) => List.cons sep (List.cons a r)) List.nil xs))))