Skip to content

Commit 507d89c

Browse files
feat: simplification lemmas for Vector.map / Vector.mapAccumr (#5558)
Primarily focused on folding nested applications of `mapAccumr` into a single `mapAccumr` Co-authored-by: Chris Hughes <chrishughes24@gmail.com>
1 parent ddfe2a5 commit 507d89c

File tree

4 files changed

+399
-6
lines changed

4 files changed

+399
-6
lines changed

Mathlib.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1795,6 +1795,7 @@ import Mathlib.Data.ULift
17951795
import Mathlib.Data.UnionFind
17961796
import Mathlib.Data.Vector
17971797
import Mathlib.Data.Vector.Basic
1798+
import Mathlib.Data.Vector.MapLemmas
17981799
import Mathlib.Data.Vector.Mem
17991800
import Mathlib.Data.Vector.Snoc
18001801
import Mathlib.Data.Vector.Zip

Mathlib/Data/Vector/Basic.lean

Lines changed: 0 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -810,8 +810,6 @@ theorem get_map₂ (v₁ : Vector α n) (v₂ : Vector β n) (f : α → β →
810810
· simp only [get_zero, head_cons]
811811
· simp only [get_cons_succ, ih]
812812

813-
814-
815813
@[simp]
816814
theorem mapAccumr_cons :
817815
mapAccumr f (x ::ᵥ xs) s

0 commit comments

Comments
 (0)