Documentation

Init.Data.List.Basic

Basic operations on List. #

We define

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:

Further operations are defined in Init.Data.List.BasicAux (because they use Array in their implementations), namely:

Preliminaries from Init.Prelude #

length #

theorem List.length_nil {α : Type u} :
theorem List.length_singleton {α : Type u} {a : α} :
theorem List.length_cons {α : Type u} {a : α} {as : List α} :
Eq (cons a as).length (HAdd.hAdd as.length 1)

set #

theorem List.length_set {α : Type u} {as : List α} {i : Nat} {a : α} :
Eq (as.set i a).length as.length

foldl #

theorem List.foldl_nil {α✝ : Type u_1} {β✝ : Type u_2} {f : α✝β✝α✝} {b : α✝} :
Eq (foldl f b nil) b
theorem List.foldl_cons {α : Type u} {β : Type v} {a : α} {l : List α} {f : βαβ} {b : β} :
Eq (foldl f b (cons a l)) (foldl f (f b a) l)

concat #

theorem List.length_concat {α : Type u} {as : List α} {a : α} :
theorem List.of_concat_eq_concat {α : Type u} {as bs : List α} {a b : α} (h : Eq (as.concat a) (bs.concat b)) :
And (Eq as bs) (Eq a b)

Equality #

def List.beq {α : Type u} [BEq α] :
List αList αBool

Checks whether two lists have the same length and their elements are pairwise BEq. Normally used via the == operator.

Equations
Instances For
    theorem List.beq_cons_nil {α : Type u} [BEq α] {a : α} {as : List α} :
    theorem List.beq_nil_cons {α : Type u} [BEq α] {a : α} {as : List α} :
    theorem List.beq_cons₂ {α : Type u} [BEq α] {a b : α} {as bs : List α} :
    Eq ((cons a as).beq (cons b bs)) ((BEq.beq a b).and (as.beq bs))
    def List.instBEq {α : Type u} [BEq α] :
    BEq (List α)
    Equations
    Instances For
      theorem List.instLawfulBEq {α : Type u} [BEq α] [LawfulBEq α] :
      @[specialize #[]]
      def List.isEqv {α : Type u} (as bs : List α) (eqv : ααBool) :

      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
        theorem List.isEqv_nil_nil {α : Type u} {eqv : ααBool} :
        theorem List.isEqv_nil_cons {α : Type u} {a : α} {as : List α} {eqv : ααBool} :
        Eq (nil.isEqv (cons a as) eqv) Bool.false
        theorem List.isEqv_cons_nil {α : Type u} {a : α} {as : List α} {eqv : ααBool} :
        Eq ((cons a as).isEqv nil eqv) Bool.false
        theorem List.isEqv_cons₂ {α✝ : Type u_1} {a : α✝} {as : List α✝} {b : α✝} {bs : List α✝} {eqv : α✝α✝Bool} :
        Eq ((cons a as).isEqv (cons b bs) eqv) ((eqv a b).and (as.isEqv bs eqv))

        Lexicographic ordering #

        inductive List.Lex {α : Type u} (r : ααProp) (as bs : List α) :

        Lexicographic ordering for lists with respect to an ordering of elements.

        as is lexicographically smaller than bs if

        • as is empty and bs is non-empty, or
        • both as and bs are non-empty, and the head of as is less than the head of bs according to r, or
        • both as and bs are non-empty, their heads are equal, and the tail of as is less than the tail of bs.
        • 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
          def List.decidableLex {α : Type u} [DecidableEq α] (r : ααProp) [h : DecidableRel r] (l₁ l₂ : List α) :
          Decidable (Lex r l₁ l₂)
          Instances For
            @[reducible, inline]
            abbrev List.lt {α : Type u} [LT α] :
            List αList αProp

            Lexicographic ordering of lists with respect to an ordering on their elements.

            as < bs if

            • as is empty and bs is non-empty, or
            • both as and bs are non-empty, and the head of as is less than the head of bs, or
            • both as and bs are non-empty, their heads are equal, and the tail of as is less than the tail of bs.
            Equations
            Instances For
              def List.instLT {α : Type u} [LT α] :
              LT (List α)
              Equations
              Instances For
                def List.decidableLT {α : Type u} [DecidableEq α] [LT α] [DecidableLT α] (l₁ l₂ : List α) :
                Decidable (LT.lt l₁ l₂)

                Decidability of lexicographic ordering.

                Equations
                Instances For
                  @[reducible, inline, deprecated List.decidableLT (since := "2024-12-13")]
                  abbrev List.hasDecidableLt {α : Type u_1} [DecidableEq α] [LT α] [DecidableLT α] (l₁ l₂ : List α) :
                  Decidable (LT.lt l₁ l₂)

                  Decidability of lexicographic ordering.

                  Equations
                  Instances For
                    @[reducible]
                    def List.le {α : Type u} [LT α] (as bs : List α) :

                    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 and bs are non-empty, and the head of as is less than the head of bs, or
                    • both as and bs are non-empty, their heads are equal, and the tail of as is less than or equal to the tail of bs.
                    Equations
                    Instances For
                      def List.instLE {α : Type u} [LT α] :
                      LE (List α)
                      Equations
                      Instances For
                        def List.decidableLE {α : Type u} [DecidableEq α] [LT α] [DecidableLT α] (l₁ l₂ : List α) :
                        Decidable (LE.le l₁ l₂)
                        Equations
                        Instances For
                          def List.lex {α : Type u} [BEq α] (l₁ l₂ : List α) (lt : ααBool := by exact (· < ·)) :

                          Compares lists lexicographically with respect to a comparison on their elements.

                          The lexicographic order with respect to lt is:

                          • [].lex (b :: bs) is true
                          • as.lex [] = false is false
                          • (a :: as).lex (b :: bs) is true if lt a b or a == b and lex lt as bs is true.
                          Equations
                          Instances For
                            theorem List.nil_lex_nil {α : Type u} {lt : ααBool} [BEq α] :
                            theorem List.nil_lex_cons {α : Type u} {lt : ααBool} [BEq α] {b : α} {bs : List α} :
                            Eq (nil.lex (cons b bs) lt) Bool.true
                            theorem List.cons_lex_nil {α : Type u} {lt : ααBool} [BEq α] {a : α} {as : List α} :
                            Eq ((cons a as).lex nil lt) Bool.false
                            theorem List.cons_lex_cons {α : Type u} {lt : ααBool} [BEq α] {a b : α} {as bs : List α} :
                            Eq ((cons a as).lex (cons b bs) lt) ((lt a b).or ((BEq.beq a b).and (as.lex bs lt)))
                            theorem List.lex_nil {α : Type u} {lt : ααBool} [BEq α] {as : List α} :
                            @[deprecated List.nil_lex_nil (since := "2025-02-10")]
                            theorem List.lex_nil_nil {α : Type u} {lt : ααBool} [BEq α] :
                            @[deprecated List.nil_lex_cons (since := "2025-02-10")]
                            theorem List.lex_nil_cons {α : Type u} {lt : ααBool} [BEq α] {b : α} {bs : List α} :
                            Eq (nil.lex (cons b bs) lt) Bool.true
                            @[deprecated List.cons_lex_nil (since := "2025-02-10")]
                            theorem List.lex_cons_nil {α : Type u} {lt : ααBool} [BEq α] {a : α} {as : List α} :
                            Eq ((cons a as).lex nil lt) Bool.false
                            @[deprecated List.cons_lex_cons (since := "2025-02-10")]
                            theorem List.lex_cons_cons {α : Type u} {lt : ααBool} [BEq α] {a b : α} {as bs : List α} :
                            Eq ((cons a as).lex (cons b bs) lt) ((lt a b).or ((BEq.beq a b).and (as.lex bs lt)))

                            Alternative getters #

                            getLast #

                            def List.getLast {α : Type u} (as : List α) :
                            Ne as nilα

                            Returns the last element of a non-empty list.

                            Examples:

                            • ["circle", "rectangle"].getLast (by decide) = "rectangle"
                            • ["circle"].getLast (by decide) = "circle"
                            Equations
                            Instances For

                              getLast? #

                              def List.getLast? {α : Type u} :
                              List αOption α

                              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:

                              Equations
                              Instances For

                                getLastD #

                                def List.getLastD {α : Type u} (as : List α) (fallback : α) :
                                α

                                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:

                                Equations
                                Instances For
                                  theorem List.getLastD_nil {α : Type u} {a : α} :
                                  theorem List.getLastD_cons {α : Type u} {a b : α} {l : List α} :
                                  Eq ((cons b l).getLastD a) (l.getLastD b)

                                  Head and tail #

                                  def List.head {α : Type u} (as : List α) :
                                  Ne as nilα

                                  Returns the first element of a non-empty list.

                                  Equations
                                  Instances For
                                    theorem List.head_cons {α : Type u} {a : α} {l : List α} {h : Ne (cons a l) nil} :
                                    Eq ((cons a l).head h) a
                                    def List.head? {α : Type u} :
                                    List αOption α

                                    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
                                    Instances For
                                      theorem List.head?_cons {α : Type u} {a : α} {l : List α} :

                                      headD #

                                      def List.headD {α : Type u} (as : List α) (fallback : α) :
                                      α

                                      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:

                                      • [].headD "empty" = "empty"
                                      • [].headD 2 = 2
                                      • ["head", "shoulders", "knees"].headD "toes" = "head"
                                      Equations
                                      Instances For
                                        theorem List.headD_nil {α : Type u} {d : α} :
                                        Eq (nil.headD d) d
                                        theorem List.headD_cons {α : Type u} {a : α} {l : List α} {d : α} :
                                        Eq ((cons a l).headD d) a

                                        tail #

                                        def List.tail {α : Type u} :
                                        List αList α

                                        Drops the first element of a nonempty list, returning the tail. Returns [] when the argument is empty.

                                        Examples:

                                        • ["apple", "banana", "grape"].tail = ["banana", "grape"]
                                        • ["apple"].tail = []
                                        • ([] : List String).tail = []
                                        Equations
                                        Instances For
                                          theorem List.tail_cons {α : Type u} {a : α} {as : List α} :
                                          Eq (cons a as).tail as

                                          tail? #

                                          def List.tail? {α : Type u} :
                                          List αOption (List α)

                                          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
                                          Instances For
                                            theorem List.tail?_cons {α : Type u} {a : α} {l : List α} :

                                            tailD #

                                            def List.tailD {α : Type u} (l fallback : List α) :
                                            List α

                                            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
                                              theorem List.tailD_nil {α : Type u} {l' : List α} :
                                              Eq (nil.tailD l') l'
                                              theorem List.tailD_cons {α : Type u} {a : α} {l l' : List α} :
                                              Eq ((cons a l).tailD l') l

                                              Basic List operations. #

                                              We define the basic functional programming operations on List: map, filter, filterMap, foldr, append, flatten, pure, bind, replicate, and reverse.

                                              map #

                                              @[specialize #[]]
                                              def List.map {α : Type u} {β : Type v} (f : αβ) (l : List α) :
                                              List β

                                              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
                                                theorem List.map_nil {α : Type u} {β : Type v} {f : αβ} :
                                                theorem List.map_cons {α : Type u} {β : Type v} {f : αβ} {a : α} {l : List α} :
                                                Eq (map f (cons a l)) (cons (f a) (map f l))

                                                filter #

                                                def List.filter {α : Type u} (p : αBool) (l : List α) :
                                                List α

                                                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
                                                Instances For
                                                  theorem List.filter_nil {α : Type u} {p : αBool} :

                                                  filterMap #

                                                  @[specialize #[]]
                                                  def List.filterMap {α : Type u} {β : Type v} (f : αOption β) :
                                                  List αList β

                                                  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
                                                  Instances For
                                                    theorem List.filterMap_nil {α : Type u} {β : Type v} {f : αOption β} :
                                                    theorem List.filterMap_cons {α : Type u} {β : Type v} {f : αOption β} {a : α} {l : List α} :
                                                    Eq (filterMap f (cons a l)) (filterMap.match_1 (fun (x : Option β) => List β) (f a) (fun (_ : Unit) => filterMap f l) fun (b : β) => cons b (filterMap f l))

                                                    foldr #

                                                    @[specialize #[]]
                                                    def List.foldr {α : Type u} {β : Type v} (f : αββ) (init : β) (l : List α) :
                                                    β

                                                    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
                                                    Instances For
                                                      theorem List.foldr_nil {α✝ : Type u_1} {α✝¹ : Type u_2} {f : α✝α✝¹α✝¹} {b : α✝¹} :
                                                      Eq (foldr f b nil) b
                                                      theorem List.foldr_cons {α : Type u} {β : Type v} {a : α} {l : List α} {f : αββ} {b : β} :
                                                      Eq (foldr f b (cons a l)) (f a (foldr f b l))

                                                      reverse #

                                                      def List.reverseAux {α : Type u} :
                                                      List αList αList α

                                                      Auxiliary for List.reverse. List.reverseAux l r = l.reverse ++ r, but it is defined directly.

                                                      Equations
                                                      Instances For
                                                        theorem List.reverseAux_nil {α✝ : Type u_1} {r : List α✝} :
                                                        theorem List.reverseAux_cons {α✝ : Type u_1} {a : α✝} {l r : List α✝} :
                                                        Eq ((cons a l).reverseAux r) (l.reverseAux (cons a r))
                                                        def List.reverse {α : Type u} (as : List α) :
                                                        List α

                                                        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
                                                        Instances For
                                                          theorem List.reverseAux_reverseAux {α : Type u} {as bs cs : List α} :

                                                          append #

                                                          def List.append {α : Type u} (xs ys : List α) :
                                                          List α

                                                          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].
                                                          Equations
                                                          Instances For
                                                            def List.appendTR {α : Type u} (as bs : List α) :
                                                            List α

                                                            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
                                                            Instances For
                                                              def List.instAppend {α : Type u} :
                                                              Equations
                                                              Instances For
                                                                theorem List.append_eq {α : Type u} {as bs : List α} :
                                                                Eq (as.append bs) (HAppend.hAppend as bs)
                                                                theorem List.nil_append {α : Type u} (as : List α) :
                                                                theorem List.cons_append {α : Type u} {a : α} {as bs : List α} :
                                                                Eq (HAppend.hAppend (cons a as) bs) (cons a (HAppend.hAppend as bs))
                                                                theorem List.append_nil {α : Type u} (as : List α) :
                                                                theorem List.length_append {α : Type u} {as bs : List α} :
                                                                theorem List.append_assoc {α : Type u} (as bs cs : List α) :
                                                                theorem List.instAssociativeHAppend {α : Type u} :
                                                                Std.Associative fun (x1 x2 : List α) => HAppend.hAppend x1 x2
                                                                theorem List.append_cons {α : Type u} (as : List α) (b : α) (bs : List α) :
                                                                theorem List.concat_eq_append {α : Type u} {as : List α} {a : α} :
                                                                Eq (as.concat a) (HAppend.hAppend as (cons a nil))
                                                                theorem List.reverseAux_eq_append {α : Type u} {as bs : List α} :
                                                                theorem List.reverse_cons {α : Type u} {a : α} {as : List α} :

                                                                flatten #

                                                                def List.flatten {α : Type u} :
                                                                List (List α)List α

                                                                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
                                                                  theorem List.flatten_cons {α✝ : Type u_1} {l : List α✝} {L : List (List α✝)} :
                                                                  @[reducible, inline, deprecated List.flatten (since := "2024-10-14")]
                                                                  abbrev List.join {α : Type u_1} :
                                                                  List (List α)List α

                                                                  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 #

                                                                    @[inline]
                                                                    def List.singleton {α : Type u} (a : α) :
                                                                    List α

                                                                    Constructs a single-element list.

                                                                    Examples:

                                                                    Equations
                                                                    Instances For
                                                                      @[reducible, inline, deprecated Singleton.singleton (since := "2024-10-16")]
                                                                      abbrev List.pure {α : outParam (Type u_1)} {β : Type u_2} [self : Singleton α β] :
                                                                      αβ
                                                                      Equations
                                                                      Instances For

                                                                        flatMap #

                                                                        @[inline]
                                                                        def List.flatMap {α : Type u} {β : Type v} (b : αList β) (as : List α) :
                                                                        List β

                                                                        Applies a function that returns a list to each element of a list, and concatenates the resulting lists.

                                                                        Examples:

                                                                        Equations
                                                                        Instances For
                                                                          theorem List.flatMap_nil {α : Type u} {β : Type v} {f : αList β} :
                                                                          theorem List.flatMap_cons {α : Type u} {β : Type v} {x : α} {xs : List α} {f : αList β} :
                                                                          Eq (flatMap f (cons x xs)) (HAppend.hAppend (f x) (flatMap f xs))
                                                                          @[reducible, inline, deprecated List.flatMap (since := "2024-10-16")]
                                                                          abbrev List.bind {α : Type u_1} {β : Type u_2} (b : αList β) (as : List α) :
                                                                          List β
                                                                          Equations
                                                                          Instances For
                                                                            @[reducible, inline, deprecated List.flatMap_nil (since := "2024-10-16")]
                                                                            abbrev List.nil_flatMap {α : Type u_1} {β : Type u_2} {f : αList β} :
                                                                            Equations
                                                                            Instances For
                                                                              @[reducible, inline, deprecated List.flatMap_cons (since := "2024-10-16")]
                                                                              abbrev List.cons_flatMap {α : Type u_1} {β : Type u_2} {x : α} {xs : List α} {f : αList β} :
                                                                              Eq (flatMap f (cons x xs)) (HAppend.hAppend (f x) (flatMap f xs))
                                                                              Equations
                                                                              Instances For

                                                                                replicate #

                                                                                def List.replicate {α : Type u} (n : Nat) (a : α) :
                                                                                List α

                                                                                Creates a list that contains n copies of a.

                                                                                Equations
                                                                                Instances For
                                                                                  theorem List.replicate_zero {α : Type u} {a : α} :
                                                                                  theorem List.replicate_succ {α : Type u} {a : α} {n : Nat} :
                                                                                  Eq (replicate (HAdd.hAdd n 1) a) (cons a (replicate n a))
                                                                                  theorem List.length_replicate {α : Type u} {n : Nat} {a : α} :

                                                                                  Additional functions #

                                                                                  leftpad and rightpad #

                                                                                  def List.leftpad {α : Type u} (n : Nat) (a : α) (l : List α) :
                                                                                  List α

                                                                                  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
                                                                                  Instances For
                                                                                    def List.rightpad {α : Type u} (n : Nat) (a : α) (l : List α) :
                                                                                    List α

                                                                                    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
                                                                                    Instances For

                                                                                      reduceOption #

                                                                                      @[inline]
                                                                                      def List.reduceOption {α : Type u_1} :
                                                                                      List (Option α)List α

                                                                                      Drop nones from a list, and replace each remaining some a with a.

                                                                                      Equations
                                                                                      Instances For

                                                                                        List membership #

                                                                                        EmptyCollection #

                                                                                        Equations
                                                                                        Instances For

                                                                                          isEmpty #

                                                                                          def List.isEmpty {α : Type u} :
                                                                                          List αBool

                                                                                          Checks whether a list is empty.

                                                                                          O(1).

                                                                                          Examples:

                                                                                          Equations
                                                                                          Instances For
                                                                                            theorem List.isEmpty_cons {α : Type u} {x : α} {xs : List α} :

                                                                                            elem #

                                                                                            def List.elem {α : Type u} [BEq α] (a : α) (l : List α) :

                                                                                            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
                                                                                              theorem List.elem_nil {α : Type u} {a : α} [BEq α] :
                                                                                              theorem List.elem_cons {α : Type u} {b : α} {bs : List α} [BEq α] {a : α} :
                                                                                              Eq (elem a (cons b bs)) (filter.match_1 (fun (x : Bool) => Bool) (BEq.beq a b) (fun (_ : Unit) => Bool.true) fun (_ : Unit) => elem a bs)

                                                                                              contains #

                                                                                              @[reducible, inline]
                                                                                              abbrev List.contains {α : Type u} [BEq α] (as : List α) (a : α) :

                                                                                              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:

                                                                                              Equations
                                                                                              Instances For
                                                                                                theorem List.contains_nil {α : Type u} {a : α} [BEq α] :

                                                                                                Mem #

                                                                                                inductive List.Mem {α : Type u} (a : α) :
                                                                                                List αProp

                                                                                                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 asMem 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
                                                                                                  def List.instMembership {α : Type u} :
                                                                                                  Equations
                                                                                                  Instances For
                                                                                                    theorem List.mem_of_elem_eq_true {α : Type u} [BEq α] [LawfulBEq α] {a : α} {as : List α} :
                                                                                                    theorem List.elem_eq_true_of_mem {α : Type u} [BEq α] [LawfulBEq α] {a : α} {as : List α} (h : Membership.mem as a) :
                                                                                                    theorem List.mem_append_left {α : Type u} {a : α} {as : List α} (bs : List α) :
                                                                                                    theorem List.mem_append_right {α : Type u} {b : α} (as : List α) {bs : List α} :
                                                                                                    def List.decidableBEx {α : Type u} (p : αProp) [DecidablePred p] (l : List α) :
                                                                                                    Decidable (Exists fun (x : α) => And (Membership.mem l x) (p x))
                                                                                                    Equations
                                                                                                    • One or more equations did not get rendered due to their size.
                                                                                                    Instances For
                                                                                                      def List.decidableBAll {α : Type u} (p : αProp) [DecidablePred p] (l : List α) :
                                                                                                      Decidable (∀ (x : α), Membership.mem l xp x)
                                                                                                      Equations
                                                                                                      • One or more equations did not get rendered due to their size.
                                                                                                      Instances For

                                                                                                        Sublists #

                                                                                                        take #

                                                                                                        def List.take {α : Type u} (n : Nat) (xs : List α) :
                                                                                                        List α

                                                                                                        Extracts the first n elements of xs, or the whole list if n is greater than xs.length.

                                                                                                        O(min n |xs|).

                                                                                                        Examples:

                                                                                                        • [a, b, c, d, e].take 0 = []
                                                                                                        • [a, b, c, d, e].take 3 = [a, b, c]
                                                                                                        • [a, b, c, d, e].take 6 = [a, b, c, d, e]
                                                                                                        Equations
                                                                                                        Instances For
                                                                                                          theorem List.take_nil {α : Type u} {i : Nat} :
                                                                                                          theorem List.take_zero {α : Type u} {l : List α} :
                                                                                                          Eq (take 0 l) nil
                                                                                                          theorem List.take_succ_cons {α : Type u} {a : α} {as : List α} {i : Nat} :
                                                                                                          Eq (take (HAdd.hAdd i 1) (cons a as)) (cons a (take i as))

                                                                                                          drop #

                                                                                                          def List.drop {α : Type u} (n : Nat) (xs : List α) :
                                                                                                          List α

                                                                                                          Removes the first n elements of the list xs. Returns the empty list if n is greater than the length of the list.

                                                                                                          O(min n |xs|).

                                                                                                          Examples:

                                                                                                          • [0, 1, 2, 3, 4].drop 0 = [0, 1, 2, 3, 4]
                                                                                                          • [0, 1, 2, 3, 4].drop 3 = [3, 4]
                                                                                                          • [0, 1, 2, 3, 4].drop 6 = []
                                                                                                          Equations
                                                                                                          Instances For
                                                                                                            theorem List.drop_nil {α : Type u} {i : Nat} :
                                                                                                            theorem List.drop_zero {α : Type u} {l : List α} :
                                                                                                            Eq (drop 0 l) l
                                                                                                            theorem List.drop_succ_cons {α : Type u} {a : α} {l : List α} {i : Nat} :
                                                                                                            Eq (drop (HAdd.hAdd i 1) (cons a l)) (drop i l)
                                                                                                            theorem List.drop_eq_nil_of_le {α : Type u} {as : List α} {i : Nat} (h : LE.le as.length i) :
                                                                                                            Eq (drop i as) nil

                                                                                                            extract #

                                                                                                            @[reducible, inline]
                                                                                                            abbrev List.extract {α : Type u} (l : List α) (start : Nat := 0) (stop : Nat := l.length) :
                                                                                                            List α

                                                                                                            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]
                                                                                                            Equations
                                                                                                            Instances For
                                                                                                              theorem List.extract_eq_drop_take {α : Type u} {l : List α} {start stop : Nat} :
                                                                                                              Eq (l.extract start stop) (take (HSub.hSub stop start) (drop start l))

                                                                                                              takeWhile #

                                                                                                              def List.takeWhile {α : Type u} (p : αBool) (xs : List α) :
                                                                                                              List α

                                                                                                              Returns the longest initial segment of xs for which p returns true.

                                                                                                              O(|xs|).

                                                                                                              Examples:

                                                                                                              Equations
                                                                                                              Instances For
                                                                                                                theorem List.takeWhile_nil {α : Type u} {p : αBool} :

                                                                                                                dropWhile #

                                                                                                                def List.dropWhile {α : Type u} (p : αBool) :
                                                                                                                List αList α

                                                                                                                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
                                                                                                                Instances For
                                                                                                                  theorem List.dropWhile_nil {α : Type u} {p : αBool} :

                                                                                                                  partition #

                                                                                                                  @[inline]
                                                                                                                  def List.partition {α : Type u} (p : αBool) (as : List α) :
                                                                                                                  Prod (List α) (List α)

                                                                                                                  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
                                                                                                                  Instances For
                                                                                                                    @[specialize #[]]
                                                                                                                    def List.partition.loop {α : Type u} (p : αBool) :
                                                                                                                    List αProd (List α) (List α)Prod (List α) (List α)
                                                                                                                    Equations
                                                                                                                    Instances For

                                                                                                                      dropLast #

                                                                                                                      def List.dropLast {α : Type u_1} :
                                                                                                                      List αList α

                                                                                                                      Removes the last element of the list, if one exists.

                                                                                                                      Examples:

                                                                                                                      Equations
                                                                                                                      Instances For
                                                                                                                        theorem List.dropLast_single {α✝ : Type u_1} {x : α✝} :
                                                                                                                        theorem List.dropLast_cons₂ {α✝ : Type u_1} {x y : α✝} {zs : List α✝} :
                                                                                                                        Eq (cons x (cons y zs)).dropLast (cons x (cons y zs).dropLast)
                                                                                                                        theorem List.length_dropLast_cons {α : Type u} {a : α} {as : List α} :

                                                                                                                        Subset #

                                                                                                                        def List.Subset {α : Type u} (l₁ l₂ : List α) :

                                                                                                                        l₁ ⊆ l₂ means that every element of l₁ is also an element of l₂, ignoring multiplicity.

                                                                                                                        Equations
                                                                                                                        Instances For
                                                                                                                          Equations
                                                                                                                          Instances For

                                                                                                                            Sublist and isSublist #

                                                                                                                            inductive List.Sublist {α : Type u_1} :
                                                                                                                            List αList αProp

                                                                                                                            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 of l₂, then it is also a subsequence of a :: 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 of l₂, then a :: l₁ is a subsequence of a :: 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
                                                                                                                              Instances For
                                                                                                                                def List.isSublist {α : Type u} [BEq α] :
                                                                                                                                List αList αBool

                                                                                                                                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? #

                                                                                                                                  def List.IsPrefix {α : Type u} (l₁ l₂ : List α) :

                                                                                                                                  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 is prefix (not isPrefix).
                                                                                                                                  Equations
                                                                                                                                  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 is prefix (not isPrefix).
                                                                                                                                    Equations
                                                                                                                                    Instances For
                                                                                                                                      def List.isPrefixOf {α : Type u} [BEq α] :
                                                                                                                                      List αList αBool

                                                                                                                                      Checks whether the first list is a prefix of the second.

                                                                                                                                      The relation List.IsPrefixOf expresses this property with respect to logical equality.

                                                                                                                                      Examples:

                                                                                                                                      Equations
                                                                                                                                      Instances For
                                                                                                                                        theorem List.isPrefixOf_cons_nil {α : Type u} {a : α} {as : List α} [BEq α] :
                                                                                                                                        theorem List.isPrefixOf_cons₂ {α : Type u} {as : List α} {b : α} {bs : List α} [BEq α] {a : α} :
                                                                                                                                        Eq ((cons a as).isPrefixOf (cons b bs)) ((BEq.beq a b).and (as.isPrefixOf bs))
                                                                                                                                        def List.isPrefixOf? {α : Type u} [BEq α] (l₁ l₂ : List α) :

                                                                                                                                        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:

                                                                                                                                        Instances For

                                                                                                                                          IsSuffix / isSuffixOf / isSuffixOf? #

                                                                                                                                          def List.isSuffixOf {α : Type u} [BEq α] (l₁ l₂ : List α) :

                                                                                                                                          Checks whether the first list is a suffix of the second.

                                                                                                                                          The relation List.IsSuffixOf expresses this property with respect to logical equality.

                                                                                                                                          Examples:

                                                                                                                                          Equations
                                                                                                                                          Instances For
                                                                                                                                            def List.isSuffixOf? {α : Type u} [BEq α] (l₁ l₂ : List α) :

                                                                                                                                            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:

                                                                                                                                            Equations
                                                                                                                                            Instances For
                                                                                                                                              def List.IsSuffix {α : Type u} (l₁ l₂ : List α) :

                                                                                                                                              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 is suffix (not isSuffix).
                                                                                                                                              Equations
                                                                                                                                              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 is suffix (not isSuffix).
                                                                                                                                                Equations
                                                                                                                                                Instances For

                                                                                                                                                  IsInfix #

                                                                                                                                                  def List.IsInfix {α : Type u} (l₁ l₂ : List α) :

                                                                                                                                                  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 is infix (not isInfix).
                                                                                                                                                  Equations
                                                                                                                                                  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 is infix (not isInfix).
                                                                                                                                                    Equations
                                                                                                                                                    Instances For

                                                                                                                                                      splitAt #

                                                                                                                                                      def List.splitAt {α : Type u} (n : Nat) (l : List α) :
                                                                                                                                                      Prod (List α) (List α)

                                                                                                                                                      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
                                                                                                                                                      Instances For
                                                                                                                                                        def List.splitAt.go {α : Type u} (l : List α) :
                                                                                                                                                        List αNatList αProd (List α) (List α)

                                                                                                                                                        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
                                                                                                                                                        Instances For

                                                                                                                                                          rotateLeft #

                                                                                                                                                          def List.rotateLeft {α : Type u} (xs : List α) (i : Nat := 1) :
                                                                                                                                                          List α

                                                                                                                                                          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:

                                                                                                                                                          Equations
                                                                                                                                                          Instances For
                                                                                                                                                            theorem List.rotateLeft_nil {α : Type u} {n : Nat} :

                                                                                                                                                            rotateRight #

                                                                                                                                                            def List.rotateRight {α : Type u} (xs : List α) (i : Nat := 1) :
                                                                                                                                                            List α

                                                                                                                                                            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:

                                                                                                                                                            Equations
                                                                                                                                                            Instances For

                                                                                                                                                              Pairwise, Nodup #

                                                                                                                                                              inductive List.Pairwise {α : Type u} (R : ααProp) :
                                                                                                                                                              List αProp

                                                                                                                                                              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:

                                                                                                                                                              • 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 lPairwise R (List.cons a l)

                                                                                                                                                                A nonempty list is pairwise related with R if the head is related to every element of the tail and the tail is itself pairwise related.

                                                                                                                                                                That is, a :: l is Pairwise R if:

                                                                                                                                                                • R relates a to every element of l
                                                                                                                                                                • l is Pairwise R.
                                                                                                                                                              Instances For
                                                                                                                                                                theorem List.pairwise_cons {α : Type u} {R : ααProp} {a : α} {l : List α} :
                                                                                                                                                                Iff (Pairwise R (cons a l)) (And (∀ (a' : α), Membership.mem l a'R a a') (Pairwise R l))
                                                                                                                                                                def List.instDecidablePairwise {α : Type u} {R : ααProp} [DecidableRel R] (l : List α) :
                                                                                                                                                                Equations
                                                                                                                                                                • One or more equations did not get rendered due to their size.
                                                                                                                                                                Instances For
                                                                                                                                                                  def List.Nodup {α : Type u} :
                                                                                                                                                                  List αProp

                                                                                                                                                                  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
                                                                                                                                                                  Instances For

                                                                                                                                                                    Manipulating elements #

                                                                                                                                                                    replace #

                                                                                                                                                                    def List.replace {α : Type u} [BEq α] (l : List α) (a b : α) :
                                                                                                                                                                    List α

                                                                                                                                                                    Replaces the first element of the list l that is equal to a with b. If no element is equal to a, then the list is returned unchanged.

                                                                                                                                                                    O(|l|).

                                                                                                                                                                    Examples:

                                                                                                                                                                    • [1, 4, 2, 3, 3, 7].replace 3 6 = [1, 4, 2, 6, 3, 7]
                                                                                                                                                                    • [1, 4, 2, 3, 3, 7].replace 5 6 = [1, 4, 2, 3, 3, 7]
                                                                                                                                                                    Equations
                                                                                                                                                                    Instances For
                                                                                                                                                                      theorem List.replace_nil {α : Type u} {a b : α} [BEq α] :
                                                                                                                                                                      theorem List.replace_cons {α : Type u} {as : List α} {b c : α} [BEq α] {a : α} :
                                                                                                                                                                      Eq ((cons a as).replace b c) (filter.match_1 (fun (x : Bool) => List α) (BEq.beq b a) (fun (_ : Unit) => cons c as) fun (_ : Unit) => cons a (as.replace b c))

                                                                                                                                                                      modify #

                                                                                                                                                                      def List.modifyTailIdx {α : Type u} (l : List α) (i : Nat) (f : List αList α) :
                                                                                                                                                                      List α

                                                                                                                                                                      Replaces the nth 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
                                                                                                                                                                      Instances For
                                                                                                                                                                        def List.modifyTailIdx.go {α : Type u} (f : List αList α) :
                                                                                                                                                                        NatList αList α
                                                                                                                                                                        Instances For
                                                                                                                                                                          theorem List.modifyTailIdx_zero {α : Type u} {f : List αList α} {l : List α} :
                                                                                                                                                                          Eq (l.modifyTailIdx 0 f) (f l)
                                                                                                                                                                          theorem List.modifyTailIdx_succ_nil {α : Type u} {f : List αList α} {i : Nat} :
                                                                                                                                                                          theorem List.modifyTailIdx_succ_cons {α : Type u} {f : List αList α} {i : Nat} {a : α} {l : List α} :
                                                                                                                                                                          Eq ((cons a l).modifyTailIdx (HAdd.hAdd i 1) f) (cons a (l.modifyTailIdx i f))
                                                                                                                                                                          @[inline]
                                                                                                                                                                          def List.modifyHead {α : Type u} (f : αα) :
                                                                                                                                                                          List αList α

                                                                                                                                                                          Replace the head of the list with the result of applying f to it. Returns the empty list if the list is empty.

                                                                                                                                                                          Examples:

                                                                                                                                                                          Equations
                                                                                                                                                                          Instances For
                                                                                                                                                                            theorem List.modifyHead_nil {α : Type u} {f : αα} :
                                                                                                                                                                            theorem List.modifyHead_cons {α : Type u} {a : α} {l : List α} {f : αα} :
                                                                                                                                                                            Eq (modifyHead f (cons a l)) (cons (f a) l)
                                                                                                                                                                            def List.modify {α : Type u} (l : List α) (i : Nat) (f : αα) :
                                                                                                                                                                            List α

                                                                                                                                                                            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
                                                                                                                                                                            Instances For

                                                                                                                                                                              insert #

                                                                                                                                                                              @[inline]
                                                                                                                                                                              def List.insert {α : Type u} [BEq α] (a : α) (l : List α) :
                                                                                                                                                                              List α

                                                                                                                                                                              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:

                                                                                                                                                                              • [1, 2, 3].insert 0 = [0, 1, 2, 3]
                                                                                                                                                                              • [1, 2, 3].insert 4 = [4, 1, 2, 3]
                                                                                                                                                                              • [1, 2, 3].insert 2 = [1, 2, 3]
                                                                                                                                                                              Equations
                                                                                                                                                                              Instances For
                                                                                                                                                                                def List.insertIdx {α : Type u} (xs : List α) (i : Nat) (a : α) :
                                                                                                                                                                                List α

                                                                                                                                                                                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
                                                                                                                                                                                Instances For

                                                                                                                                                                                  erase #

                                                                                                                                                                                  def List.erase {α : Type u_1} [BEq α] :
                                                                                                                                                                                  List ααList α

                                                                                                                                                                                  Removes the first occurrence of a from l. If a does not occur in l, the list is returned unmodified.

                                                                                                                                                                                  O(|l|).

                                                                                                                                                                                  Examples:

                                                                                                                                                                                  • [1, 5, 3, 2, 5].erase 5 = [1, 3, 2, 5]
                                                                                                                                                                                  • [1, 5, 3, 2, 5].erase 6 = [1, 5, 3, 2, 5]
                                                                                                                                                                                  Equations
                                                                                                                                                                                  Instances For
                                                                                                                                                                                    theorem List.erase_nil {α : Type u} [BEq α] (a : α) :
                                                                                                                                                                                    theorem List.erase_cons {α : Type u} [BEq α] {a b : α} {l : List α} :
                                                                                                                                                                                    Eq ((cons b l).erase a) (ite (Eq (BEq.beq b a) Bool.true) l (cons b (l.erase a)))
                                                                                                                                                                                    def List.eraseP {α : Type u} (p : αBool) :
                                                                                                                                                                                    List αList α

                                                                                                                                                                                    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
                                                                                                                                                                                    Instances For

                                                                                                                                                                                      eraseIdx #

                                                                                                                                                                                      def List.eraseIdx {α : Type u} (l : List α) (i : Nat) :
                                                                                                                                                                                      List α

                                                                                                                                                                                      Removes the element at the specified index. If the index is out of bounds, the list is returned unmodified.

                                                                                                                                                                                      O(i).

                                                                                                                                                                                      Examples:

                                                                                                                                                                                      • [0, 1, 2, 3, 4].eraseIdx 0 = [1, 2, 3, 4]
                                                                                                                                                                                      • [0, 1, 2, 3, 4].eraseIdx 1 = [0, 2, 3, 4]
                                                                                                                                                                                      • [0, 1, 2, 3, 4].eraseIdx 5 = [0, 1, 2, 3, 4]
                                                                                                                                                                                      Equations
                                                                                                                                                                                      Instances For
                                                                                                                                                                                        theorem List.eraseIdx_nil {α : Type u} {i : Nat} :
                                                                                                                                                                                        theorem List.eraseIdx_cons_zero {α✝ : Type u_1} {a : α✝} {as : List α✝} :
                                                                                                                                                                                        Eq ((cons a as).eraseIdx 0) as
                                                                                                                                                                                        theorem List.eraseIdx_cons_succ {α✝ : Type u_1} {a : α✝} {as : List α✝} {i : Nat} :
                                                                                                                                                                                        Eq ((cons a as).eraseIdx (HAdd.hAdd i 1)) (cons a (as.eraseIdx i))

                                                                                                                                                                                        Finding elements

                                                                                                                                                                                        find? #

                                                                                                                                                                                        def List.find? {α : Type u} (p : αBool) :
                                                                                                                                                                                        List αOption α

                                                                                                                                                                                        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:

                                                                                                                                                                                        • [7, 6, 5, 8, 1, 2, 6].find? (· < 5) = some 1
                                                                                                                                                                                        • [7, 6, 5, 8, 1, 2, 6].find? (· < 1) = none
                                                                                                                                                                                        Equations
                                                                                                                                                                                        Instances For
                                                                                                                                                                                          theorem List.find?_nil {α : Type u} {p : αBool} :
                                                                                                                                                                                          theorem List.find?_cons {α✝ : Type u_1} {a : α✝} {as : List α✝} {p : α✝Bool} :
                                                                                                                                                                                          Eq (find? p (cons a as)) (filter.match_1 (fun (x : Bool) => Option α✝) (p a) (fun (_ : Unit) => Option.some a) fun (_ : Unit) => find? p as)

                                                                                                                                                                                          findSome? #

                                                                                                                                                                                          def List.findSome? {α : Type u} {β : Type v} (f : αOption β) :
                                                                                                                                                                                          List αOption β

                                                                                                                                                                                          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
                                                                                                                                                                                          Instances For
                                                                                                                                                                                            theorem List.findSome?_nil {α : Type u} {α✝ : Type u_1} {f : αOption α✝} :
                                                                                                                                                                                            theorem List.findSome?_cons {α : Type u} {β : Type v} {a : α} {as : List α} {f : αOption β} :
                                                                                                                                                                                            Eq (findSome? f (cons a as)) (findSome?.match_1 (fun (x : Option β) => Option β) (f a) (fun (b : β) => Option.some b) fun (_ : Unit) => findSome? f as)

                                                                                                                                                                                            findIdx #

                                                                                                                                                                                            @[inline]
                                                                                                                                                                                            def List.findIdx {α : Type u} (p : αBool) (l : List α) :

                                                                                                                                                                                            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:

                                                                                                                                                                                            • [7, 6, 5, 8, 1, 2, 6].findIdx (· < 5) = 4
                                                                                                                                                                                            • [7, 6, 5, 8, 1, 2, 6].findIdx (· < 1) = 7
                                                                                                                                                                                            Equations
                                                                                                                                                                                            Instances For
                                                                                                                                                                                              @[specialize #[]]
                                                                                                                                                                                              def List.findIdx.go {α : Type u} (p : αBool) :
                                                                                                                                                                                              List αNatNat

                                                                                                                                                                                              Auxiliary for findIdx: findIdx.go p l n = findIdx p l + n

                                                                                                                                                                                              Equations
                                                                                                                                                                                              Instances For
                                                                                                                                                                                                theorem List.findIdx_nil {α : Type u} {p : αBool} :
                                                                                                                                                                                                Eq (findIdx p nil) 0

                                                                                                                                                                                                idxOf #

                                                                                                                                                                                                def List.idxOf {α : Type u} [BEq α] (a : α) :
                                                                                                                                                                                                List αNat

                                                                                                                                                                                                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
                                                                                                                                                                                                Instances For
                                                                                                                                                                                                  @[reducible, inline, deprecated List.idxOf (since := "2025-01-29")]
                                                                                                                                                                                                  abbrev List.indexOf {α : Type u_1} [BEq α] (a : α) :
                                                                                                                                                                                                  List αNat

                                                                                                                                                                                                  Returns the index of the first element equal to a, or the length of the list otherwise.

                                                                                                                                                                                                  Equations
                                                                                                                                                                                                  Instances For
                                                                                                                                                                                                    theorem List.idxOf_nil {α : Type u} {x : α} [BEq α] :
                                                                                                                                                                                                    Eq (idxOf x nil) 0
                                                                                                                                                                                                    @[deprecated List.idxOf_nil (since := "2025-01-29")]
                                                                                                                                                                                                    theorem List.indexOf_nil {α : Type u} {x : α} [BEq α] :
                                                                                                                                                                                                    Eq (idxOf x nil) 0

                                                                                                                                                                                                    findIdx? #

                                                                                                                                                                                                    def List.findIdx? {α : Type u} (p : αBool) (l : List α) :

                                                                                                                                                                                                    Returns the index of the first element for which p returns true, or none if there is no such element.

                                                                                                                                                                                                    Examples:

                                                                                                                                                                                                    • [7, 6, 5, 8, 1, 2, 6].findIdx (· < 5) = some 4
                                                                                                                                                                                                    • [7, 6, 5, 8, 1, 2, 6].findIdx (· < 1) = none
                                                                                                                                                                                                    Equations
                                                                                                                                                                                                    Instances For
                                                                                                                                                                                                      def List.findIdx?.go {α : Type u} (p : αBool) :
                                                                                                                                                                                                      List αNatOption Nat
                                                                                                                                                                                                      Equations
                                                                                                                                                                                                      Instances For

                                                                                                                                                                                                        idxOf? #

                                                                                                                                                                                                        @[inline]
                                                                                                                                                                                                        def List.idxOf? {α : Type u} [BEq α] (a : α) :
                                                                                                                                                                                                        List αOption Nat

                                                                                                                                                                                                        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
                                                                                                                                                                                                        Instances For
                                                                                                                                                                                                          @[reducible, inline, deprecated List.idxOf? (since := "2025-01-29")]
                                                                                                                                                                                                          abbrev List.indexOf? {α : Type u_1} [BEq α] (a : α) :
                                                                                                                                                                                                          List αOption Nat

                                                                                                                                                                                                          Return the index of the first occurrence of a in the list.

                                                                                                                                                                                                          Equations
                                                                                                                                                                                                          Instances For

                                                                                                                                                                                                            findFinIdx? #

                                                                                                                                                                                                            @[inline]
                                                                                                                                                                                                            def List.findFinIdx? {α : Type u} (p : αBool) (l : List α) :

                                                                                                                                                                                                            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:

                                                                                                                                                                                                            Equations
                                                                                                                                                                                                            Instances For
                                                                                                                                                                                                              def List.findFinIdx?.go {α : Type u} (p : αBool) (l l' : List α) (i : Nat) (h : Eq (HAdd.hAdd l'.length i) l.length) :
                                                                                                                                                                                                              Equations
                                                                                                                                                                                                              Instances For

                                                                                                                                                                                                                finIdxOf? #

                                                                                                                                                                                                                @[inline]
                                                                                                                                                                                                                def List.finIdxOf? {α : Type u} [BEq α] (a : α) (l : List α) :

                                                                                                                                                                                                                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
                                                                                                                                                                                                                Instances For

                                                                                                                                                                                                                  countP #

                                                                                                                                                                                                                  @[inline]
                                                                                                                                                                                                                  def List.countP {α : Type u} (p : αBool) (l : List α) :

                                                                                                                                                                                                                  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
                                                                                                                                                                                                                  Instances For
                                                                                                                                                                                                                    @[specialize #[]]
                                                                                                                                                                                                                    def List.countP.go {α : Type u} (p : αBool) :
                                                                                                                                                                                                                    List αNatNat

                                                                                                                                                                                                                    Auxiliary for countP: countP.go p l acc = countP p l + acc.

                                                                                                                                                                                                                    Equations
                                                                                                                                                                                                                    Instances For

                                                                                                                                                                                                                      count #

                                                                                                                                                                                                                      @[inline]
                                                                                                                                                                                                                      def List.count {α : Type u} [BEq α] (a : α) :
                                                                                                                                                                                                                      List αNat

                                                                                                                                                                                                                      Counts the number of times an element occurs in a list.

                                                                                                                                                                                                                      Examples:

                                                                                                                                                                                                                      • [1, 1, 2, 3, 5].count 1 = 2
                                                                                                                                                                                                                      • [1, 1, 2, 3, 5].count 5 = 1
                                                                                                                                                                                                                      • [1, 1, 2, 3, 5].count 4 = 0
                                                                                                                                                                                                                      Equations
                                                                                                                                                                                                                      Instances For

                                                                                                                                                                                                                        lookup #

                                                                                                                                                                                                                        def List.lookup {α : Type u} {β : Type v} [BEq α] :
                                                                                                                                                                                                                        αList (Prod α β)Option β

                                                                                                                                                                                                                        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
                                                                                                                                                                                                                          theorem List.lookup_nil {α : Type u} {β : Type v} {a : α} [BEq α] :
                                                                                                                                                                                                                          theorem List.lookup_cons {α : Type u} {β✝ : Type u_1} {b : β✝} {as : List (Prod α β✝)} {a : α} [BEq α] {k : α} :
                                                                                                                                                                                                                          Eq (lookup a (cons { fst := k, snd := b } as)) (filter.match_1 (fun (x : Bool) => Option β✝) (BEq.beq a k) (fun (_ : Unit) => Option.some b) fun (_ : Unit) => lookup a as)

                                                                                                                                                                                                                          Permutations #

                                                                                                                                                                                                                          Perm #

                                                                                                                                                                                                                          inductive List.Perm {α : Type u} :
                                                                                                                                                                                                                          List αList αProp

                                                                                                                                                                                                                          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
                                                                                                                                                                                                                            Instances For

                                                                                                                                                                                                                              isPerm #

                                                                                                                                                                                                                              def List.isPerm {α : Type u} [BEq α] :
                                                                                                                                                                                                                              List αList αBool

                                                                                                                                                                                                                              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 #

                                                                                                                                                                                                                                def List.any {α : Type u} (l : List α) (p : αBool) :

                                                                                                                                                                                                                                Returns true if p returns true for any element of l.

                                                                                                                                                                                                                                O(|l|). Short-circuits upon encountering the first true.

                                                                                                                                                                                                                                Examples:

                                                                                                                                                                                                                                • [2, 4, 6].any (· % 2 = 0) = true
                                                                                                                                                                                                                                • [2, 4, 6].any (· % 2 = 1) = false
                                                                                                                                                                                                                                • [2, 4, 5, 6].any (· % 2 = 0) = true
                                                                                                                                                                                                                                • [2, 4, 5, 6].any (· % 2 = 1) = true
                                                                                                                                                                                                                                Equations
                                                                                                                                                                                                                                Instances For
                                                                                                                                                                                                                                  theorem List.any_nil {α✝ : Type u_1} {f : α✝Bool} :
                                                                                                                                                                                                                                  theorem List.any_cons {α✝ : Type u_1} {a : α✝} {l : List α✝} {f : α✝Bool} :
                                                                                                                                                                                                                                  Eq ((cons a l).any f) ((f a).or (l.any f))

                                                                                                                                                                                                                                  all #

                                                                                                                                                                                                                                  def List.all {α : Type u} :
                                                                                                                                                                                                                                  List α(αBool)Bool

                                                                                                                                                                                                                                  Returns true if p returns true for every element of l.

                                                                                                                                                                                                                                  O(|l|). Short-circuits upon encountering the first false.

                                                                                                                                                                                                                                  Examples:

                                                                                                                                                                                                                                  • [a, b, c].all p = (p a && (p b && p c))
                                                                                                                                                                                                                                  • [2, 4, 6].all (· % 2 = 0) = true
                                                                                                                                                                                                                                  • [2, 4, 5, 6].all (· % 2 = 0) = false
                                                                                                                                                                                                                                  Equations
                                                                                                                                                                                                                                  Instances For
                                                                                                                                                                                                                                    theorem List.all_nil {α✝ : Type u_1} {f : α✝Bool} :
                                                                                                                                                                                                                                    theorem List.all_cons {α✝ : Type u_1} {a : α✝} {l : List α✝} {f : α✝Bool} :
                                                                                                                                                                                                                                    Eq ((cons a l).all f) ((f a).and (l.all f))

                                                                                                                                                                                                                                    or #

                                                                                                                                                                                                                                    def List.or (bs : List Bool) :

                                                                                                                                                                                                                                    Returns true if true is an element of the list bs.

                                                                                                                                                                                                                                    O(|bs|). Short-circuits at the first true value.

                                                                                                                                                                                                                                    • [true, true, true].or = true
                                                                                                                                                                                                                                    • [true, false, true].or = true
                                                                                                                                                                                                                                    • [false, false, false].or = false
                                                                                                                                                                                                                                    • [false, false, true].or = true
                                                                                                                                                                                                                                    • [].or = false
                                                                                                                                                                                                                                    Equations
                                                                                                                                                                                                                                    Instances For
                                                                                                                                                                                                                                      theorem List.or_cons {a : Bool} {l : List Bool} :
                                                                                                                                                                                                                                      Eq (cons a l).or (a.or l.or)

                                                                                                                                                                                                                                      and #

                                                                                                                                                                                                                                      def List.and (bs : List Bool) :

                                                                                                                                                                                                                                      Returns true if every element of bs is the value true.

                                                                                                                                                                                                                                      O(|bs|). Short-circuits at the first false value.

                                                                                                                                                                                                                                      • [true, true, true].and = true
                                                                                                                                                                                                                                      • [true, false, true].and = false
                                                                                                                                                                                                                                      • [true, false, false].and = false
                                                                                                                                                                                                                                      • [].and = true
                                                                                                                                                                                                                                      Equations
                                                                                                                                                                                                                                      Instances For
                                                                                                                                                                                                                                        theorem List.and_cons {a : Bool} {l : List Bool} :
                                                                                                                                                                                                                                        Eq (cons a l).and (a.and l.and)

                                                                                                                                                                                                                                        Zippers #

                                                                                                                                                                                                                                        zipWith #

                                                                                                                                                                                                                                        @[specialize #[]]
                                                                                                                                                                                                                                        def List.zipWith {α : Type u} {β : Type v} {γ : Type w} (f : αβγ) (xs : List α) (ys : List β) :
                                                                                                                                                                                                                                        List γ

                                                                                                                                                                                                                                        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
                                                                                                                                                                                                                                        Instances For
                                                                                                                                                                                                                                          theorem List.zipWith_nil_left {α : Type u} {β : Type v} {γ : Type w} {l : List β} {f : αβγ} :
                                                                                                                                                                                                                                          theorem List.zipWith_nil_right {α : Type u} {β : Type v} {γ : Type w} {l : List α} {f : αβγ} :
                                                                                                                                                                                                                                          theorem List.zipWith_cons_cons {α : Type u} {β : Type v} {γ : Type w} {a : α} {as : List α} {b : β} {bs : List β} {f : αβγ} :
                                                                                                                                                                                                                                          Eq (zipWith f (cons a as) (cons b bs)) (cons (f a b) (zipWith f as bs))

                                                                                                                                                                                                                                          zip #

                                                                                                                                                                                                                                          def List.zip {α : Type u} {β : Type v} :
                                                                                                                                                                                                                                          List αList βList (Prod α β)

                                                                                                                                                                                                                                          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
                                                                                                                                                                                                                                            theorem List.zip_nil_left {α : Type u} {β : Type v} {l : List β} :
                                                                                                                                                                                                                                            theorem List.zip_nil_right {α : Type u} {β : Type v} {l : List α} :
                                                                                                                                                                                                                                            theorem List.zip_cons_cons {α✝ : Type u_1} {a : α✝} {as : List α✝} {α✝¹ : Type u_2} {b : α✝¹} {bs : List α✝¹} :
                                                                                                                                                                                                                                            Eq ((cons a as).zip (cons b bs)) (cons { fst := a, snd := b } (as.zip bs))

                                                                                                                                                                                                                                            zipWithAll #

                                                                                                                                                                                                                                            def List.zipWithAll {α : Type u} {β : Type v} {γ : Type w} (f : Option αOption βγ) :
                                                                                                                                                                                                                                            List αList βList γ

                                                                                                                                                                                                                                            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
                                                                                                                                                                                                                                              theorem List.zipWithAll_nil {α✝ : Type u_1} {α✝¹ : Type u_2} {α✝² : Type u_3} {f : Option α✝Option α✝¹α✝²} {as : List α✝} :
                                                                                                                                                                                                                                              Eq (zipWithAll f as nil) (map (fun (a : α✝) => f (Option.some a) Option.none) as)
                                                                                                                                                                                                                                              theorem List.nil_zipWithAll {α✝ : Type u_1} {α✝¹ : Type u_2} {α✝² : Type u_3} {f : Option α✝Option α✝¹α✝²} {bs : List α✝¹} :
                                                                                                                                                                                                                                              Eq (zipWithAll f nil bs) (map (fun (b : α✝¹) => f Option.none (Option.some b)) bs)
                                                                                                                                                                                                                                              theorem List.zipWithAll_cons_cons {α✝ : Type u_1} {α✝¹ : Type u_2} {α✝² : Type u_3} {f : Option α✝Option α✝¹α✝²} {a : α✝} {as : List α✝} {b : α✝¹} {bs : List α✝¹} :
                                                                                                                                                                                                                                              Eq (zipWithAll f (cons a as) (cons b bs)) (cons (f (Option.some a) (Option.some b)) (zipWithAll f as bs))

                                                                                                                                                                                                                                              unzip #

                                                                                                                                                                                                                                              def List.unzip {α : Type u} {β : Type v} (l : List (Prod α β)) :
                                                                                                                                                                                                                                              Prod (List α) (List β)

                                                                                                                                                                                                                                              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
                                                                                                                                                                                                                                                theorem List.unzip_nil {α : Type u} {β : Type v} :
                                                                                                                                                                                                                                                Eq nil.unzip { fst := nil, snd := nil }
                                                                                                                                                                                                                                                theorem List.unzip_cons {α : Type u} {β : Type v} {t : List (Prod α β)} {h : Prod α β} :
                                                                                                                                                                                                                                                Eq (cons h t).unzip (unzip.match_1 (fun (x : Prod (List α) (List β)) => Prod (List α) (List β)) t.unzip fun (as : List α) (bs : List β) => { fst := cons h.fst as, snd := cons h.snd bs })

                                                                                                                                                                                                                                                Ranges and enumeration #

                                                                                                                                                                                                                                                def List.sum {α : Type u_1} [Add α] [Zero α] :
                                                                                                                                                                                                                                                List αα

                                                                                                                                                                                                                                                Computes the sum of the elements of a list.

                                                                                                                                                                                                                                                Examples:

                                                                                                                                                                                                                                                • [a, b, c].sum = a + (b + (c + 0))
                                                                                                                                                                                                                                                • [1, 2, 5].sum = 8
                                                                                                                                                                                                                                                Equations
                                                                                                                                                                                                                                                Instances For
                                                                                                                                                                                                                                                  theorem List.sum_nil {α : Type u} [Add α] [Zero α] :
                                                                                                                                                                                                                                                  theorem List.sum_cons {α : Type u} [Add α] [Zero α] {a : α} {l : List α} :
                                                                                                                                                                                                                                                  Eq (cons a l).sum (HAdd.hAdd a l.sum)
                                                                                                                                                                                                                                                  @[deprecated List.sum (since := "2024-10-17")]
                                                                                                                                                                                                                                                  def Nat.sum (l : List Nat) :

                                                                                                                                                                                                                                                  Sum of a list of natural numbers.

                                                                                                                                                                                                                                                  Equations
                                                                                                                                                                                                                                                  Instances For
                                                                                                                                                                                                                                                    @[deprecated List.sum_nil (since := "2024-10-17")]
                                                                                                                                                                                                                                                    @[deprecated List.sum_cons (since := "2024-10-17")]
                                                                                                                                                                                                                                                    theorem Nat.sum_cons (a : Nat) (l : List Nat) :

                                                                                                                                                                                                                                                    range #

                                                                                                                                                                                                                                                    def List.range (n : Nat) :

                                                                                                                                                                                                                                                    Returns a list of the numbers from 0 to n exclusive, in increasing order.

                                                                                                                                                                                                                                                    O(n).

                                                                                                                                                                                                                                                    Examples:

                                                                                                                                                                                                                                                    Equations
                                                                                                                                                                                                                                                    Instances For
                                                                                                                                                                                                                                                      Equations
                                                                                                                                                                                                                                                      • One or more equations did not get rendered due to their size.
                                                                                                                                                                                                                                                      Instances For

                                                                                                                                                                                                                                                        range' #

                                                                                                                                                                                                                                                        def List.range' (start len : Nat) (step : Nat := 1) :

                                                                                                                                                                                                                                                        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:

                                                                                                                                                                                                                                                        Equations
                                                                                                                                                                                                                                                        Instances For

                                                                                                                                                                                                                                                          iota #

                                                                                                                                                                                                                                                          @[deprecated "Use `(List.range' 1 n).reverse` instead of `iota n`." (since := "2025-01-20")]

                                                                                                                                                                                                                                                          O(n). iota n is the numbers from 1 to n inclusive, in decreasing order.

                                                                                                                                                                                                                                                          • iota 5 = [5, 4, 3, 2, 1]
                                                                                                                                                                                                                                                          Equations
                                                                                                                                                                                                                                                          Instances For
                                                                                                                                                                                                                                                            theorem List.iota_succ {i : Nat} :
                                                                                                                                                                                                                                                            Eq (iota (HAdd.hAdd i 1)) (cons (HAdd.hAdd i 1) (iota i))

                                                                                                                                                                                                                                                            zipIdx #

                                                                                                                                                                                                                                                            def List.zipIdx {α : Type u} (l : List α) (n : Nat := 0) :

                                                                                                                                                                                                                                                            Pairs each element of a list with its index, optionally starting from an index other than 0.

                                                                                                                                                                                                                                                            O(|l|).

                                                                                                                                                                                                                                                            Examples:

                                                                                                                                                                                                                                                            • [a, b, c].zipIdx = [(a, 0), (b, 1), (c, 2)]
                                                                                                                                                                                                                                                            • [a, b, c].zipIdx 5 = [(a, 5), (b, 6), (c, 7)]
                                                                                                                                                                                                                                                            Equations
                                                                                                                                                                                                                                                            Instances For
                                                                                                                                                                                                                                                              theorem List.zipIdx_nil {α : Type u} {i : Nat} :
                                                                                                                                                                                                                                                              theorem List.zipIdx_cons {α✝ : Type u_1} {a : α✝} {as : List α✝} {i : Nat} :
                                                                                                                                                                                                                                                              Eq ((cons a as).zipIdx i) (cons { fst := a, snd := i } (as.zipIdx (HAdd.hAdd i 1)))

                                                                                                                                                                                                                                                              enumFrom #

                                                                                                                                                                                                                                                              @[deprecated "Use `zipIdx` instead; note the signature change." (since := "2025-01-21")]
                                                                                                                                                                                                                                                              def List.enumFrom {α : Type u} :
                                                                                                                                                                                                                                                              NatList αList (Prod Nat α)

                                                                                                                                                                                                                                                              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
                                                                                                                                                                                                                                                              Instances For
                                                                                                                                                                                                                                                                @[deprecated List.zipIdx_nil (since := "2025-01-21")]
                                                                                                                                                                                                                                                                theorem List.enumFrom_nil {α : Type u} {i : Nat} :
                                                                                                                                                                                                                                                                @[deprecated List.zipIdx_cons (since := "2025-01-21")]
                                                                                                                                                                                                                                                                theorem List.enumFrom_cons {α✝ : Type u_1} {a : α✝} {as : List α✝} {i : Nat} :
                                                                                                                                                                                                                                                                Eq (enumFrom i (cons a as)) (cons { fst := i, snd := a } (enumFrom (HAdd.hAdd i 1) as))

                                                                                                                                                                                                                                                                enum #

                                                                                                                                                                                                                                                                @[deprecated "Use `zipIdx` instead; note the signature change." (since := "2025-01-21")]
                                                                                                                                                                                                                                                                def List.enum {α : Type u} :
                                                                                                                                                                                                                                                                List αList (Prod Nat α)

                                                                                                                                                                                                                                                                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
                                                                                                                                                                                                                                                                Instances For
                                                                                                                                                                                                                                                                  @[deprecated List.zipIdx_nil (since := "2025-01-21")]
                                                                                                                                                                                                                                                                  theorem List.enum_nil {α : Type u} :

                                                                                                                                                                                                                                                                  Minima and maxima #

                                                                                                                                                                                                                                                                  min? #

                                                                                                                                                                                                                                                                  def List.min? {α : Type u} [Min α] :
                                                                                                                                                                                                                                                                  List αOption α

                                                                                                                                                                                                                                                                  Returns the smallest element of the list if it is not empty, or none if it is empty.

                                                                                                                                                                                                                                                                  Examples:

                                                                                                                                                                                                                                                                  • [].min? = none
                                                                                                                                                                                                                                                                  • [4].min? = some 4
                                                                                                                                                                                                                                                                  • [1, 4, 2, 10, 6].min? = some 1
                                                                                                                                                                                                                                                                  Equations
                                                                                                                                                                                                                                                                  Instances For
                                                                                                                                                                                                                                                                    @[reducible, inline, deprecated List.min? (since := "2024-09-29")]
                                                                                                                                                                                                                                                                    abbrev List.minimum? {α : Type u_1} [Min α] :
                                                                                                                                                                                                                                                                    List αOption α

                                                                                                                                                                                                                                                                    Returns the smallest element of the list if it is not empty, or none if it is empty.

                                                                                                                                                                                                                                                                    Examples:

                                                                                                                                                                                                                                                                    • [].min? = none
                                                                                                                                                                                                                                                                    • [4].min? = some 4
                                                                                                                                                                                                                                                                    • [1, 4, 2, 10, 6].min? = some 1
                                                                                                                                                                                                                                                                    Equations
                                                                                                                                                                                                                                                                    Instances For

                                                                                                                                                                                                                                                                      max? #

                                                                                                                                                                                                                                                                      def List.max? {α : Type u} [Max α] :
                                                                                                                                                                                                                                                                      List αOption α

                                                                                                                                                                                                                                                                      Returns the largest element of the list if it is not empty, or none if it is empty.

                                                                                                                                                                                                                                                                      Examples:

                                                                                                                                                                                                                                                                      • [].max? = none
                                                                                                                                                                                                                                                                      • [4].max? = some 4
                                                                                                                                                                                                                                                                      • [1, 4, 2, 10, 6].max? = some 10
                                                                                                                                                                                                                                                                      Equations
                                                                                                                                                                                                                                                                      Instances For
                                                                                                                                                                                                                                                                        @[reducible, inline, deprecated List.max? (since := "2024-09-29")]
                                                                                                                                                                                                                                                                        abbrev List.maximum? {α : Type u_1} [Max α] :
                                                                                                                                                                                                                                                                        List αOption α

                                                                                                                                                                                                                                                                        Returns the largest element of the list if it is not empty, or none if it is empty.

                                                                                                                                                                                                                                                                        Examples:

                                                                                                                                                                                                                                                                        • [].max? = none
                                                                                                                                                                                                                                                                        • [4].max? = some 4
                                                                                                                                                                                                                                                                        • [1, 4, 2, 10, 6].max? = some 10
                                                                                                                                                                                                                                                                        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 #

                                                                                                                                                                                                                                                                          def List.intersperse {α : Type u} (sep : α) (l : List α) :
                                                                                                                                                                                                                                                                          List α

                                                                                                                                                                                                                                                                          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:

                                                                                                                                                                                                                                                                          Equations
                                                                                                                                                                                                                                                                          Instances For
                                                                                                                                                                                                                                                                            theorem List.intersperse_nil {α : Type u} {sep : α} :
                                                                                                                                                                                                                                                                            theorem List.intersperse_single {α : Type u} {x sep : α} :
                                                                                                                                                                                                                                                                            Eq (intersperse sep (cons x nil)) (cons x nil)
                                                                                                                                                                                                                                                                            theorem List.intersperse_cons₂ {α : Type u} {x y : α} {zs : List α} {sep : α} :
                                                                                                                                                                                                                                                                            Eq (intersperse sep (cons x (cons y zs))) (cons x (cons sep (intersperse sep (cons y zs))))

                                                                                                                                                                                                                                                                            intercalate #

                                                                                                                                                                                                                                                                            def List.intercalate {α : Type u} (sep : List α) (xs : List (List α)) :
                                                                                                                                                                                                                                                                            List α

                                                                                                                                                                                                                                                                            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:

                                                                                                                                                                                                                                                                            Equations
                                                                                                                                                                                                                                                                            Instances For

                                                                                                                                                                                                                                                                              eraseDups #

                                                                                                                                                                                                                                                                              def List.eraseDups {α : Type u_1} [BEq α] (as : List α) :
                                                                                                                                                                                                                                                                              List α

                                                                                                                                                                                                                                                                              Erases duplicated elements in the list, keeping the first occurrence of duplicated elements.

                                                                                                                                                                                                                                                                              O(|l|^2).

                                                                                                                                                                                                                                                                              Examples:

                                                                                                                                                                                                                                                                              • [1, 3, 2, 2, 3, 5].eraseDups = [1, 3, 2, 5]
                                                                                                                                                                                                                                                                              • ["red", "green", "green", "blue"].eraseDups = ["red", "green", "blue"]
                                                                                                                                                                                                                                                                              Equations
                                                                                                                                                                                                                                                                              Instances For
                                                                                                                                                                                                                                                                                def List.eraseDups.loop {α : Type u_1} [BEq α] :
                                                                                                                                                                                                                                                                                List αList αList α
                                                                                                                                                                                                                                                                                Equations
                                                                                                                                                                                                                                                                                • One or more equations did not get rendered due to their size.
                                                                                                                                                                                                                                                                                Instances For

                                                                                                                                                                                                                                                                                  eraseReps #

                                                                                                                                                                                                                                                                                  def List.eraseReps {α : Type u_1} [BEq α] :
                                                                                                                                                                                                                                                                                  List αList α

                                                                                                                                                                                                                                                                                  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
                                                                                                                                                                                                                                                                                  Instances For
                                                                                                                                                                                                                                                                                    def List.eraseReps.loop {α : Type u_1} [BEq α] :
                                                                                                                                                                                                                                                                                    αList αList αList α
                                                                                                                                                                                                                                                                                    Equations
                                                                                                                                                                                                                                                                                    • One or more equations did not get rendered due to their size.
                                                                                                                                                                                                                                                                                    Instances For

                                                                                                                                                                                                                                                                                      span #

                                                                                                                                                                                                                                                                                      @[inline]
                                                                                                                                                                                                                                                                                      def List.span {α : Type u} (p : αBool) (as : List α) :
                                                                                                                                                                                                                                                                                      Prod (List α) (List α)

                                                                                                                                                                                                                                                                                      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
                                                                                                                                                                                                                                                                                      Instances For
                                                                                                                                                                                                                                                                                        @[specialize #[]]
                                                                                                                                                                                                                                                                                        def List.span.loop {α : Type u} (p : αBool) :
                                                                                                                                                                                                                                                                                        List αList αProd (List α) (List α)
                                                                                                                                                                                                                                                                                        Equations
                                                                                                                                                                                                                                                                                        • One or more equations did not get rendered due to their size.
                                                                                                                                                                                                                                                                                        Instances For

                                                                                                                                                                                                                                                                                          splitBy #

                                                                                                                                                                                                                                                                                          @[specialize #[]]
                                                                                                                                                                                                                                                                                          def List.splitBy {α : Type u} (R : ααBool) :
                                                                                                                                                                                                                                                                                          List αList (List α)

                                                                                                                                                                                                                                                                                          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
                                                                                                                                                                                                                                                                                            @[specialize #[]]
                                                                                                                                                                                                                                                                                            def List.splitBy.loop {α : Type u} (R : ααBool) :
                                                                                                                                                                                                                                                                                            List ααList αList (List α)List (List α)

                                                                                                                                                                                                                                                                                            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
                                                                                                                                                                                                                                                                                              @[reducible, inline, deprecated List.splitBy (since := "2024-10-30")]
                                                                                                                                                                                                                                                                                              abbrev List.groupBy {α : Type u_1} (R : ααBool) :
                                                                                                                                                                                                                                                                                              List αList (List α)

                                                                                                                                                                                                                                                                                              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 #

                                                                                                                                                                                                                                                                                                def List.removeAll {α : Type u} [BEq α] (xs ys : List α) :
                                                                                                                                                                                                                                                                                                List α

                                                                                                                                                                                                                                                                                                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
                                                                                                                                                                                                                                                                                                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 #

                                                                                                                                                                                                                                                                                                  theorem List.length_add_eq_lengthTRAux {α : Type u} {as : List α} {n : Nat} :

                                                                                                                                                                                                                                                                                                  map #

                                                                                                                                                                                                                                                                                                  @[inline]
                                                                                                                                                                                                                                                                                                  def List.mapTR {α : Type u} {β : Type v} (f : αβ) (as : List α) :
                                                                                                                                                                                                                                                                                                  List β

                                                                                                                                                                                                                                                                                                  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
                                                                                                                                                                                                                                                                                                  Instances For
                                                                                                                                                                                                                                                                                                    @[specialize #[]]
                                                                                                                                                                                                                                                                                                    def List.mapTR.loop {α : Type u} {β : Type v} (f : αβ) :
                                                                                                                                                                                                                                                                                                    List αList βList β
                                                                                                                                                                                                                                                                                                    Equations
                                                                                                                                                                                                                                                                                                    Instances For
                                                                                                                                                                                                                                                                                                      theorem List.mapTR_loop_eq {α : Type u} {β : Type v} {f : αβ} {as : List α} {bs : List β} :
                                                                                                                                                                                                                                                                                                      Eq (mapTR.loop f as bs) (HAppend.hAppend bs.reverse (map f as))

                                                                                                                                                                                                                                                                                                      filter #

                                                                                                                                                                                                                                                                                                      @[inline]
                                                                                                                                                                                                                                                                                                      def List.filterTR {α : Type u} (p : αBool) (as : List α) :
                                                                                                                                                                                                                                                                                                      List α

                                                                                                                                                                                                                                                                                                      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
                                                                                                                                                                                                                                                                                                      Instances For
                                                                                                                                                                                                                                                                                                        @[specialize #[]]
                                                                                                                                                                                                                                                                                                        def List.filterTR.loop {α : Type u} (p : αBool) :
                                                                                                                                                                                                                                                                                                        List αList αList α
                                                                                                                                                                                                                                                                                                        Equations
                                                                                                                                                                                                                                                                                                        Instances For
                                                                                                                                                                                                                                                                                                          theorem List.filterTR_loop_eq {α : Type u} {p : αBool} {as bs : List α} :

                                                                                                                                                                                                                                                                                                          replicate #

                                                                                                                                                                                                                                                                                                          def List.replicateTR {α : Type u} (n : Nat) (a : α) :
                                                                                                                                                                                                                                                                                                          List α

                                                                                                                                                                                                                                                                                                          Creates a list that contains n copies of a.

                                                                                                                                                                                                                                                                                                          This is a tail-recursive version of List.replicate.

                                                                                                                                                                                                                                                                                                          Equations
                                                                                                                                                                                                                                                                                                          Instances For
                                                                                                                                                                                                                                                                                                            def List.replicateTR.loop {α : Type u} (a : α) :
                                                                                                                                                                                                                                                                                                            NatList αList α
                                                                                                                                                                                                                                                                                                            Equations
                                                                                                                                                                                                                                                                                                            Instances For
                                                                                                                                                                                                                                                                                                              theorem List.replicateTR_loop_replicate_eq {α : Type u} {a : α} {m n : Nat} :
                                                                                                                                                                                                                                                                                                              theorem List.replicateTR_loop_eq {α✝ : Type u_1} {a : α✝} {acc : List α✝} (n : Nat) :

                                                                                                                                                                                                                                                                                                              Additional functions #

                                                                                                                                                                                                                                                                                                              leftpad #

                                                                                                                                                                                                                                                                                                              @[inline]
                                                                                                                                                                                                                                                                                                              def List.leftpadTR {α : Type u} (n : Nat) (a : α) (l : List α) :
                                                                                                                                                                                                                                                                                                              List α

                                                                                                                                                                                                                                                                                                              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
                                                                                                                                                                                                                                                                                                              Instances For

                                                                                                                                                                                                                                                                                                                Zippers #

                                                                                                                                                                                                                                                                                                                unzip #

                                                                                                                                                                                                                                                                                                                def List.unzipTR {α : Type u} {β : Type v} (l : List (Prod α β)) :
                                                                                                                                                                                                                                                                                                                Prod (List α) (List β)

                                                                                                                                                                                                                                                                                                                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' #

                                                                                                                                                                                                                                                                                                                  @[inline]
                                                                                                                                                                                                                                                                                                                  def List.range'TR (s n : Nat) (step : Nat := 1) :

                                                                                                                                                                                                                                                                                                                  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:

                                                                                                                                                                                                                                                                                                                  Equations
                                                                                                                                                                                                                                                                                                                  Instances For
                                                                                                                                                                                                                                                                                                                    def List.range'TR.go (step : Nat := 1) :
                                                                                                                                                                                                                                                                                                                    NatNatList NatList Nat

                                                                                                                                                                                                                                                                                                                    Auxiliary for range'TR: range'TR.go n e = [e-n, ..., e-1] ++ acc.

                                                                                                                                                                                                                                                                                                                    Equations
                                                                                                                                                                                                                                                                                                                    Instances For
                                                                                                                                                                                                                                                                                                                      theorem List.range'_eq_range'TR.go (step : Nat := 1) (s n m : Nat) :
                                                                                                                                                                                                                                                                                                                      Eq (range'TR.go step n (HAdd.hAdd s (HMul.hMul step n)) (range' (HAdd.hAdd s (HMul.hMul step n)) m step)) (range' s (HAdd.hAdd n m) step)

                                                                                                                                                                                                                                                                                                                      iota #

                                                                                                                                                                                                                                                                                                                      @[deprecated "Use `List.range' 1 n` instead of `iota n`." (since := "2025-01-20")]
                                                                                                                                                                                                                                                                                                                      def List.iotaTR (n : Nat) :

                                                                                                                                                                                                                                                                                                                      Tail-recursive version of List.iota.

                                                                                                                                                                                                                                                                                                                      Equations
                                                                                                                                                                                                                                                                                                                      Instances For
                                                                                                                                                                                                                                                                                                                        Equations
                                                                                                                                                                                                                                                                                                                        Instances For

                                                                                                                                                                                                                                                                                                                          Other list operations #

                                                                                                                                                                                                                                                                                                                          intersperse #

                                                                                                                                                                                                                                                                                                                          def List.intersperseTR {α : Type u} (sep : α) (l : List α) :
                                                                                                                                                                                                                                                                                                                          List α

                                                                                                                                                                                                                                                                                                                          Alternates the elements of l with sep.

                                                                                                                                                                                                                                                                                                                          O(|l|).

                                                                                                                                                                                                                                                                                                                          This is a tail-recursive version of List.intersperse, used at runtime.

                                                                                                                                                                                                                                                                                                                          Examples:

                                                                                                                                                                                                                                                                                                                          Equations
                                                                                                                                                                                                                                                                                                                          Instances For