We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
ofFn_get
1 parent 09610fd commit d7a4357Copy full SHA for d7a4357
Mathlib/Data/Vector/Basic.lean
@@ -164,10 +164,8 @@ theorem get_ofFn {n} (f : Fin n → α) (i) : get (ofFn f) i = f i := by
164
165
@[simp]
166
theorem ofFn_get (v : Vector α n) : ofFn (get v) = v := by
167
- rcases v with ⟨l, rfl⟩
168
- apply toList_injective
169
- dsimp
170
- simpa only [toList_ofFn] using List.ofFn_get _
+ ext
+ apply List.Vector.get_ofFn
171
172
/-- The natural equivalence between length-`n` vectors and functions from `Fin n`. -/
173
def _root_.Equiv.vectorEquivFin (α : Type*) (n : ℕ) : Vector α n ≃ (Fin n → α) :=
0 commit comments