Commit 2024-12-15 09:21 07a54609

View on Github →

chore: rename Mathlib.Vector to List.Vector (#19930) Per @digama0's suggestion on zulip.

Estimated changes

modified def Nat.Partrec'.Vec
modified theorem Nat.Partrec'.comp₁
modified theorem Nat.Partrec'.of_eq
modified theorem Nat.Partrec'.of_prim
modified theorem Nat.Partrec'.rfindOpt
modified inductive Nat.Partrec'
modified def Nat.Primrec'.Vec
modified theorem Nat.Primrec'.of_eq
modified inductive Nat.Primrec'
modified theorem Primrec.vector_cons
modified theorem Primrec.vector_get'
modified theorem Primrec.vector_get
modified theorem Primrec.vector_head
modified theorem Primrec.vector_length
modified theorem Primrec.vector_ofFn'
modified theorem Primrec.vector_tail
modified theorem Primrec.vector_toList
modified theorem Primrec.vector_toList_iff
modified theorem Sym.cons_of_coe_eq
modified def Sym.ofVector
modified theorem Sym.ofVector_cons
modified theorem Sym.ofVector_nil
modified theorem Sym.sound
added theorem List.Vector.cons_val
added theorem List.Vector.ext
added theorem List.Vector.get_eq_get
added theorem List.Vector.get_map
added theorem List.Vector.get_ofFn
added theorem List.Vector.get_tail
added theorem List.Vector.get_zero
added theorem List.Vector.head_map
added theorem List.Vector.head_ofFn
added theorem List.Vector.head_pmap
added def List.Vector.last
added theorem List.Vector.last_def
added theorem List.Vector.length_val
added theorem List.Vector.mOfFn_pure
added theorem List.Vector.map_id
added theorem List.Vector.map₂_nil
added theorem List.Vector.mk_toList
added def List.Vector.mmap
added theorem List.Vector.mmap_cons
added theorem List.Vector.mmap_nil
added theorem List.Vector.ofFn_get
added theorem List.Vector.pmap_cons'
added theorem List.Vector.pmap_cons
added theorem List.Vector.prod_set'
added theorem List.Vector.prod_set
added theorem List.Vector.scanl_cons
added theorem List.Vector.scanl_get
added theorem List.Vector.scanl_head
added theorem List.Vector.scanl_nil
added theorem List.Vector.scanl_val
added def List.Vector.set
added theorem List.Vector.tail_map
added theorem List.Vector.tail_nil
added theorem List.Vector.tail_ofFn
added theorem List.Vector.tail_pmap
added theorem List.Vector.tail_val
added theorem List.Vector.toList_map
added theorem List.Vector.toList_set
deleted theorem Mathlib.Vector.append_nil
deleted theorem Mathlib.Vector.cons_val
deleted theorem Mathlib.Vector.ext
deleted theorem Mathlib.Vector.get_eq_get
deleted theorem Mathlib.Vector.get_map
deleted theorem Mathlib.Vector.get_map₂
deleted theorem Mathlib.Vector.get_ofFn
deleted theorem Mathlib.Vector.get_tail
deleted theorem Mathlib.Vector.get_zero
deleted theorem Mathlib.Vector.head_map
deleted theorem Mathlib.Vector.head_ofFn
deleted theorem Mathlib.Vector.head_pmap
deleted def Mathlib.Vector.last
deleted theorem Mathlib.Vector.last_def
deleted theorem Mathlib.Vector.length_val
deleted theorem Mathlib.Vector.mOfFn_pure
deleted theorem Mathlib.Vector.map_id
deleted theorem Mathlib.Vector.map₂_nil
deleted theorem Mathlib.Vector.mk_toList
deleted def Mathlib.Vector.mmap
deleted theorem Mathlib.Vector.mmap_cons
deleted theorem Mathlib.Vector.mmap_nil
deleted theorem Mathlib.Vector.ofFn_get
deleted theorem Mathlib.Vector.pmap_cons'
deleted theorem Mathlib.Vector.pmap_cons
deleted theorem Mathlib.Vector.prod_set'
deleted theorem Mathlib.Vector.prod_set
deleted theorem Mathlib.Vector.scanl_cons
deleted theorem Mathlib.Vector.scanl_get
deleted theorem Mathlib.Vector.scanl_head
deleted theorem Mathlib.Vector.scanl_nil
deleted theorem Mathlib.Vector.scanl_val
deleted def Mathlib.Vector.set
deleted theorem Mathlib.Vector.tail_map
deleted theorem Mathlib.Vector.tail_nil
deleted theorem Mathlib.Vector.tail_ofFn
deleted theorem Mathlib.Vector.tail_pmap
deleted theorem Mathlib.Vector.tail_val
deleted theorem Mathlib.Vector.toList_map
deleted theorem Mathlib.Vector.toList_set
added def List.Vector.cons
added def List.Vector.drop
added def List.Vector.elim
added def List.Vector.get
added def List.Vector.head
added theorem List.Vector.head_cons
added def List.Vector.map
added theorem List.Vector.map_cons
added theorem List.Vector.map_nil
added def List.Vector.nil
added def List.Vector.ofFn
added def List.Vector.pmap
added theorem List.Vector.pmap_nil
added def List.Vector.tail
added theorem List.Vector.tail_cons
added def List.Vector.take
added theorem List.Vector.toList_mk
added theorem List.Vector.toList_nil
added def List.Vector
deleted def Mathlib.Vector.cons
deleted def Mathlib.Vector.drop
deleted def Mathlib.Vector.elim
deleted def Mathlib.Vector.get
deleted def Mathlib.Vector.head
deleted theorem Mathlib.Vector.head_cons
deleted def Mathlib.Vector.map
deleted theorem Mathlib.Vector.map_cons
deleted theorem Mathlib.Vector.map_nil
deleted def Mathlib.Vector.nil
deleted def Mathlib.Vector.ofFn
deleted def Mathlib.Vector.pmap
deleted theorem Mathlib.Vector.pmap_nil
deleted def Mathlib.Vector.tail
deleted theorem Mathlib.Vector.tail_cons
deleted def Mathlib.Vector.take
deleted theorem Mathlib.Vector.toList_mk
deleted theorem Mathlib.Vector.toList_nil
deleted def Mathlib.Vector
added theorem List.Vector.map_map
added theorem List.Vector.map_map₂
added theorem List.Vector.map_pmap
added theorem List.Vector.pmap_map
deleted theorem Mathlib.Vector.map_map
deleted theorem Mathlib.Vector.map_map₂
deleted theorem Mathlib.Vector.map_pmap
deleted theorem Mathlib.Vector.pmap_map