Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit ec1b70e

Browse files
committed
chore(linear_algebra/multilinear): Add map_update_zero (#5417)
`map_coord_zero` isn't in a form that can be used by simp, so this introduces a form which can.
1 parent 5e057c9 commit ec1b70e

File tree

1 file changed

+3
-0
lines changed

1 file changed

+3
-0
lines changed

src/linear_algebra/multilinear.lean

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -116,6 +116,9 @@ begin
116116
rw [← update_eq_self i m, h, ← this, f.map_smul, zero_smul]
117117
end
118118

119+
@[simp] lemma map_update_zero (m : Πi, M₁ i) (i : ι) : f (update m i 0) = 0 :=
120+
f.map_coord_zero i (update_same i 0 m)
121+
119122
@[simp] lemma map_zero [nonempty ι] : f 0 = 0 :=
120123
begin
121124
obtain ⟨i, _⟩ : ∃i:ι, i ∈ set.univ := set.exists_mem_of_nonempty ι,

0 commit comments

Comments
 (0)