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

Commit ca95e36

Browse files
committed
chore(linear_algebra/basic): golf a lemma statement (#17752)
1 parent d57133e commit ca95e36

File tree

1 file changed

+2
-2
lines changed

1 file changed

+2
-2
lines changed

src/linear_algebra/basic.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1217,9 +1217,9 @@ disjoint_ker.trans
12171217
⟨λ H x hx y hy h, eq_of_sub_eq_zero $ H _ (sub_mem hx hy) (by simp [h]),
12181218
λ H x h₁ h₂, H x h₁ 0 (zero_mem _) (by simpa using h₂)⟩
12191219

1220-
theorem inj_of_disjoint_ker {p : submodule R M}
1220+
theorem inj_on_of_disjoint_ker {p : submodule R M}
12211221
{s : set M} (h : s ⊆ p) (hd : disjoint p (ker f)) :
1222-
∀ x y ∈ s, f x = f y → x = y :=
1222+
set.inj_on f s :=
12231223
λ x hx y hy, disjoint_ker'.1 hd _ (h hx) _ (h hy)
12241224

12251225
variables (F)

0 commit comments

Comments
 (0)