Documentation

Mathlib.Data.List.GetD

getD and getI #

This file provides theorems for working with the getD and getI functions. These are used to access an element of a list by numerical index, with a default value as a fallback when the index is out of range.

theorem List.getD_eq_get {α : Type u} (l : List α) (d : α) {n : } (hn : n < l.length) :
l.getD n d = l.get n, hn
@[simp]
theorem List.getD_map {α : Type u} {β : Type v} (l : List α) (d : α) {n : } (f : αβ) :
(List.map f l).getD n (f d) = f (l.getD n d)
theorem List.getD_eq_default {α : Type u} (l : List α) (d : α) {n : } (hn : l.length n) :
l.getD n d = d
def List.decidableGetDNilNe {α : Type u_1} (a : α) :
DecidablePred fun (i : ) => [].getD i a a

An empty list can always be decidably checked for the presence of an element. Not an instance because it would clash with DecidableEq α.

Equations
Instances For
    @[simp]
    theorem List.getD_singleton_default_eq {α : Type u} (d : α) (n : ) :
    [d].getD n d = d
    @[simp]
    theorem List.getD_replicate_default_eq {α : Type u} (d : α) (r : ) (n : ) :
    (List.replicate r d).getD n d = d
    theorem List.getD_append {α : Type u} (l : List α) (l' : List α) (d : α) (n : ) (h : n < l.length) :
    (l ++ l').getD n d = l.getD n d
    theorem List.getD_append_right {α : Type u} (l : List α) (l' : List α) (d : α) (n : ) (h : l.length n) :
    (l ++ l').getD n d = l'.getD (n - l.length) d
    theorem List.getD_eq_getD_get? {α : Type u} (l : List α) (d : α) (n : ) :
    l.getD n d = (l.get? n).getD d
    @[simp]
    theorem List.getI_nil {α : Type u} (n : ) [Inhabited α] :
    [].getI n = default
    @[simp]
    theorem List.getI_cons_zero {α : Type u} (x : α) (xs : List α) [Inhabited α] :
    (x :: xs).getI 0 = x
    @[simp]
    theorem List.getI_cons_succ {α : Type u} (x : α) (xs : List α) (n : ) [Inhabited α] :
    (x :: xs).getI (n + 1) = xs.getI n
    theorem List.getI_eq_get {α : Type u} (l : List α) [Inhabited α] {n : } (hn : n < l.length) :
    l.getI n = l.get n, hn
    theorem List.getI_eq_default {α : Type u} (l : List α) [Inhabited α] {n : } (hn : l.length n) :
    l.getI n = default
    theorem List.getD_default_eq_getI {α : Type u} (l : List α) [Inhabited α] {n : } :
    l.getD n default = l.getI n
    theorem List.getI_append {α : Type u} [Inhabited α] (l : List α) (l' : List α) (n : ) (h : n < l.length) :
    (l ++ l').getI n = l.getI n
    theorem List.getI_append_right {α : Type u} [Inhabited α] (l : List α) (l' : List α) (n : ) (h : l.length n) :
    (l ++ l').getI n = l'.getI (n - l.length)
    theorem List.getI_eq_iget_get? {α : Type u} (l : List α) [Inhabited α] (n : ) :
    l.getI n = (l.get? n).iget
    theorem List.getI_zero_eq_headI {α : Type u} (l : List α) [Inhabited α] :
    l.getI 0 = l.headI