Documentation

Mathlib.Data.List.Indexes

Lemmas about List.*Idx functions. #

Some specification lemmas for List.mapIdx, List.mapIdxM, List.foldlIdx and List.foldrIdx.

def List.oldMapIdxCore {α : Type u} {β : Type v} (f : αβ) :
List αList β

Lean3 map_with_index helper function

Equations
Instances For
    def List.oldMapIdx {α : Type u} {β : Type v} (f : αβ) (as : List α) :
    List β

    Given a function f : ℕ → α → β and as : List α, as = [a₀, a₁, ...], returns the list [f 0 a₀, f 1 a₁, ...].

    Equations
    Instances For
      @[simp]
      theorem List.mapIdx_nil {α : Type u_1} {β : Type u_2} (f : αβ) :
      List.mapIdx f [] = []
      theorem List.oldMapIdxCore_eq {α : Type u} {β : Type v} (l : List α) (f : αβ) (n : ) :
      List.oldMapIdxCore f n l = List.oldMapIdx (fun (i : ) (a : α) => f (i + n) a) l
      theorem List.list_reverse_induction {α : Type u} (p : List αProp) (base : p []) (ind : ∀ (l : List α) (e : α), p lp (l ++ [e])) (l : List α) :
      p l
      theorem List.oldMapIdxCore_append {α : Type u} {β : Type v} (f : αβ) (n : ) (l₁ : List α) (l₂ : List α) :
      List.oldMapIdxCore f n (l₁ ++ l₂) = List.oldMapIdxCore f n l₁ ++ List.oldMapIdxCore f (n + List.length l₁) l₂
      theorem List.oldMapIdx_append {α : Type u} {β : Type v} (f : αβ) (l : List α) (e : α) :
      theorem List.mapIdxGo_append {α : Type u} {β : Type v} (f : αβ) (l₁ : List α) (l₂ : List α) (arr : Array β) :
      List.mapIdx.go f (l₁ ++ l₂) arr = List.mapIdx.go f l₂ (List.toArray (List.mapIdx.go f l₁ arr))
      theorem List.mapIdxGo_length {α : Type u} {β : Type v} (f : αβ) (l : List α) (arr : Array β) :
      theorem List.mapIdx_append_one {α : Type u} {β : Type v} (f : αβ) (l : List α) (e : α) :
      List.mapIdx f (l ++ [e]) = List.mapIdx f l ++ [f (List.length l) e]
      theorem List.new_def_eq_old_def {α : Type u} {β : Type v} (f : αβ) (l : List α) :
      theorem List.map_enumFrom_eq_zipWith {α : Type u} {β : Type v} (l : List α) (n : ) (f : αβ) :
      theorem List.mapIdx_eq_enum_map {α : Type u} {β : Type v} (l : List α) (f : αβ) :
      @[simp]
      theorem List.mapIdx_cons {α : Type u_1} {β : Type u_2} (l : List α) (f : αβ) (a : α) :
      List.mapIdx f (a :: l) = f 0 a :: List.mapIdx (fun (i : ) => f (i + 1)) l
      theorem List.mapIdx_append {β : Type v} {α : Type u_1} (K : List α) (L : List α) (f : αβ) :
      List.mapIdx f (K ++ L) = List.mapIdx f K ++ List.mapIdx (fun (i : ) (a : α) => f (i + List.length K) a) L
      @[simp]
      theorem List.length_mapIdx {α : Type u_1} {β : Type u_2} (l : List α) (f : αβ) :
      @[simp]
      theorem List.mapIdx_eq_nil {α : Type u_1} {β : Type u_2} {f : αβ} {l : List α} :
      List.mapIdx f l = [] l = []
      @[simp, deprecated]
      theorem List.nthLe_mapIdx {α : Type u_1} {β : Type u_2} (l : List α) (f : αβ) (i : ) (h : i < List.length l) (h' : optParam (i < List.length (List.mapIdx f l)) ) :
      List.nthLe (List.mapIdx f l) i h' = f i (List.nthLe l i h)
      theorem List.mapIdx_eq_ofFn {α : Type u_1} {β : Type u_2} (l : List α) (f : αβ) :
      List.mapIdx f l = List.ofFn fun (i : Fin (List.length l)) => f (i) (List.get l i)
      def List.foldrIdxSpec {α : Type u} {β : Type v} (f : αββ) (b : β) (as : List α) (start : ) :
      β

      Specification of foldrIdx.

      Equations
      Instances For
        theorem List.foldrIdxSpec_cons {α : Type u} {β : Type v} (f : αββ) (b : β) (a : α) (as : List α) (start : ) :
        List.foldrIdxSpec f b (a :: as) start = f start a (List.foldrIdxSpec f b as (start + 1))
        theorem List.foldrIdx_eq_foldrIdxSpec {α : Type u} {β : Type v} (f : αββ) (b : β) (as : List α) (start : ) :
        List.foldrIdx f b as start = List.foldrIdxSpec f b as start
        theorem List.foldrIdx_eq_foldr_enum {α : Type u} {β : Type v} (f : αββ) (b : β) (as : List α) :
        theorem List.indexesValues_eq_filter_enum {α : Type u} (p : αProp) [DecidablePred p] (as : List α) :
        List.indexesValues (fun (b : α) => decide (p b)) as = List.filter ((fun (b : α) => decide (p b)) Prod.snd) (List.enum as)
        theorem List.findIdxs_eq_map_indexesValues {α : Type u} (p : αProp) [DecidablePred p] (as : List α) :
        List.findIdxs (fun (b : α) => decide (p b)) as = List.map Prod.fst (List.indexesValues (fun (b : α) => decide (p b)) as)
        theorem List.findIdx_eq_length {α : Type u} {p : αBool} {xs : List α} :
        List.findIdx p xs = List.length xs xxs, ¬p x = true
        theorem List.findIdx_le_length {α : Type u} (p : αBool) {xs : List α} :
        theorem List.findIdx_lt_length {α : Type u} {p : αBool} {xs : List α} :
        List.findIdx p xs < List.length xs ∃ x ∈ xs, p x = true
        theorem List.not_of_lt_findIdx {α : Type u} {p : αBool} {xs : List α} {i : } (h : i < List.findIdx p xs) :
        ¬p (List.get xs { val := i, isLt := }) = true

        p does not hold for elements with indices less than xs.findIdx p.

        theorem List.le_findIdx_of_not {α : Type u} {p : αBool} {xs : List α} {i : } (h : i < List.length xs) (h2 : ∀ (j : ) (hji : j < i), ¬p (List.get xs { val := j, isLt := }) = true) :
        theorem List.lt_findIdx_of_not {α : Type u} {p : αBool} {xs : List α} {i : } (h : i < List.length xs) (h2 : ∀ (j : ) (hji : j i), ¬p (List.get xs { val := j, isLt := }) = true) :
        theorem List.findIdx_eq {α : Type u} {p : αBool} {xs : List α} {i : } (h : i < List.length xs) :
        List.findIdx p xs = i p (List.get xs { val := i, isLt := h }) = true ∀ (j : ) (hji : j < i), ¬p (List.get xs { val := j, isLt := }) = true
        def List.foldlIdxSpec {α : Type u} {β : Type v} (f : αβα) (a : α) (bs : List β) (start : ) :
        α

        Specification of foldlIdx.

        Equations
        Instances For
          theorem List.foldlIdxSpec_cons {α : Type u} {β : Type v} (f : αβα) (a : α) (b : β) (bs : List β) (start : ) :
          List.foldlIdxSpec f a (b :: bs) start = List.foldlIdxSpec f (f start a b) bs (start + 1)
          theorem List.foldlIdx_eq_foldlIdxSpec {α : Type u} {β : Type v} (f : αβα) (a : α) (bs : List β) (start : ) :
          List.foldlIdx f a bs start = List.foldlIdxSpec f a bs start
          theorem List.foldlIdx_eq_foldl_enum {α : Type u} {β : Type v} (f : αβα) (a : α) (bs : List β) :
          List.foldlIdx f a bs = List.foldl (fun (a : α) (p : × β) => f p.1 a p.2) a (List.enum bs)
          theorem List.foldrIdxM_eq_foldrM_enum {m : Type u → Type v} [Monad m] {α : Type u_1} {β : Type u} (f : αβm β) (b : β) (as : List α) [LawfulMonad m] :
          theorem List.foldlIdxM_eq_foldlM_enum {m : Type u → Type v} [Monad m] [LawfulMonad m] {α : Type u_1} {β : Type u} (f : βαm β) (b : β) (as : List α) :
          List.foldlIdxM f b as = List.foldlM (fun (b : β) (p : × α) => f p.1 b p.2) b (List.enum as)
          def List.mapIdxMAuxSpec {m : Type u → Type v} [Monad m] {α : Type u_1} {β : Type u} (f : αm β) (start : ) (as : List α) :
          m (List β)

          Specification of mapIdxMAux.

          Equations
          Instances For
            theorem List.mapIdxMAuxSpec_cons {m : Type u → Type v} [Monad m] {α : Type u_1} {β : Type u} (f : αm β) (start : ) (a : α) (as : List α) :
            List.mapIdxMAuxSpec f start (a :: as) = Seq.seq (List.cons <$> f start a) fun (x : Unit) => List.mapIdxMAuxSpec f (start + 1) as
            theorem List.mapIdxMGo_eq_mapIdxMAuxSpec {m : Type u → Type v} [Monad m] [LawfulMonad m] {α : Type u_1} {β : Type u} (f : αm β) (arr : Array β) (as : List α) :
            List.mapIdxM.go f as arr = (fun (x : List β) => Array.toList arr ++ x) <$> List.mapIdxMAuxSpec f (Array.size arr) as
            theorem List.mapIdxM_eq_mmap_enum {m : Type u → Type v} [Monad m] [LawfulMonad m] {α : Type u_1} {β : Type u} (f : αm β) (as : List α) :
            theorem List.mapIdxMAux'_eq_mapIdxMGo {m : Type u → Type v} [Monad m] [LawfulMonad m] {α : Type u_1} (f : αm PUnit.{u + 1} ) (as : List α) (arr : Array PUnit.{u + 1} ) :
            theorem List.mapIdxM'_eq_mapIdxM {m : Type u → Type v} [Monad m] [LawfulMonad m] {α : Type u_1} (f : αm PUnit.{u + 1} ) (as : List α) :