Skip to content

Commit 71d3df6

Browse files
committed
chore(LinearIndependent): rename linearCombination lemmas (#23045)
Follow the naming convention around unnamespacing and appending `_injective` better. From Toric
1 parent 15b14b2 commit 71d3df6

File tree

4 files changed

+25
-10
lines changed

4 files changed

+25
-10
lines changed

Mathlib/LinearAlgebra/LinearIndependent/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -250,7 +250,7 @@ theorem LinearIndependent.disjoint_span_image (hv : LinearIndependent R v) {s t
250250
(hs : Disjoint s t) : Disjoint (Submodule.span R <| v '' s) (Submodule.span R <| v '' t) := by
251251
simp only [disjoint_def, Finsupp.mem_span_image_iff_linearCombination]
252252
rintro _ ⟨l₁, hl₁, rfl⟩ ⟨l₂, hl₂, H⟩
253-
rw [hv.injective_linearCombination.eq_iff] at H; subst l₂
253+
rw [hv.finsuppLinearCombination_injective.eq_iff] at H; subst l₂
254254
have : l₁ = 0 := Submodule.disjoint_def.mp (Finsupp.disjoint_supported_supported hs) _ hl₁ hl₂
255255
simp [this]
256256

Mathlib/LinearAlgebra/LinearIndependent/Defs.lean

Lines changed: 21 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -115,16 +115,31 @@ variable {R v}
115115
theorem LinearIndepOn.linearIndependent {s : Set ι} (h : LinearIndepOn R v s) :
116116
LinearIndependent R (fun x : s ↦ v x) := h
117117

118-
theorem linearIndependent_iff_injective_linearCombination :
118+
theorem linearIndependent_iff_injective_finsuppLinearCombination :
119119
LinearIndependent R v ↔ Injective (Finsupp.linearCombination R v) := Iff.rfl
120120

121-
alias ⟨LinearIndependent.injective_linearCombination, _⟩ :=
122-
linearIndependent_iff_injective_linearCombination
121+
@[deprecated (since := "2025-03-18")]
122+
alias linearIndependent_iff_injective_linearCombination :=
123+
linearIndependent_iff_injective_finsuppLinearCombination
123124

124-
theorem Fintype.linearIndependent_iff_injective [Fintype ι] :
125+
alias ⟨LinearIndependent.finsuppLinearCombination_injective, _⟩ :=
126+
linearIndependent_iff_injective_finsuppLinearCombination
127+
128+
@[deprecated (since := "2025-03-18")]
129+
alias LinearIndependent.linearCombination_injective :=
130+
LinearIndependent.finsuppLinearCombination_injective
131+
132+
theorem linearIndependent_iff_injective_fintypeLinearCombination [Fintype ι] :
125133
LinearIndependent R v ↔ Injective (Fintype.linearCombination R v) := by
126134
simp [← Finsupp.linearCombination_eq_fintype_linearCombination, LinearIndependent]
127135

136+
@[deprecated (since := "2025-03-18")]
137+
alias Fintype.linearIndependent_iff_injective :=
138+
linearIndependent_iff_injective_fintypeLinearCombination
139+
140+
alias ⟨LinearIndependent.fintypeLinearCombination_injective, _⟩ :=
141+
linearIndependent_iff_injective_fintypeLinearCombination
142+
128143
theorem LinearIndependent.injective [Nontrivial R] (hv : LinearIndependent R v) : Injective v := by
129144
simpa [comp_def]
130145
using Injective.comp hv (Finsupp.single_left_injective one_ne_zero)
@@ -245,7 +260,7 @@ theorem not_linearIndependent_iffₛ :
245260

246261
theorem Fintype.linearIndependent_iffₛ [Fintype ι] :
247262
LinearIndependent R v ↔ ∀ f g : ι → R, ∑ i, f i • v i = ∑ i, g i • v i → ∀ i, f i = g i := by
248-
simp_rw [Fintype.linearIndependent_iff_injective,
263+
simp_rw [linearIndependent_iff_injective_fintypeLinearCombination,
249264
Injective, Fintype.linearCombination_apply, funext_iff]
250265

251266
theorem Fintype.not_linearIndependent_iffₛ [Fintype ι] :
@@ -581,7 +596,7 @@ theorem linearIndependent_iff'' :
581596

582597
theorem linearIndependent_add_smul_iff {c : ι → R} {i : ι} (h₀ : c i = 0) :
583598
LinearIndependent R (v + (c · • v i)) ↔ LinearIndependent R v := by
584-
simp [linearIndependent_iff_injective_linearCombination,
599+
simp [linearIndependent_iff_injective_finsuppLinearCombination,
585600
← Finsupp.linearCombination_comp_addSingleEquiv i c h₀]
586601

587602
theorem not_linearIndependent_iff :

Mathlib/LinearAlgebra/RootSystem/Finite/g2.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -167,7 +167,7 @@ lemma allRoots_eq_map_allCoeffs :
167167

168168
lemma allRoots_nodup : (allRoots P).Nodup := by
169169
have hli : Injective (Fintype.linearCombination ℤ ![shortRoot P, longRoot P]) := by
170-
rw [← Fintype.linearIndependent_iff_injective]
170+
rw [← linearIndependent_iff_injective_fintypeLinearCombination]
171171
exact (linearIndependent_short_long P).restrict_scalars' ℤ
172172
rw [allRoots_eq_map_allCoeffs, nodup_map_iff hli]
173173
decide

Mathlib/RingTheory/AlgebraicIndependent/Basic.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -65,14 +65,14 @@ theorem algebraMap_injective : Injective (algebraMap R A) := by
6565
(MvPolynomial.C_injective _ _)
6666

6767
theorem linearIndependent : LinearIndependent R x := by
68-
rw [linearIndependent_iff_injective_linearCombination]
68+
rw [linearIndependent_iff_injective_finsuppLinearCombination]
6969
have : Finsupp.linearCombination R x =
7070
(MvPolynomial.aeval x).toLinearMap.comp (Finsupp.linearCombination R X) := by
7171
ext
7272
simp
7373
rw [this]
7474
refine (algebraicIndependent_iff_injective_aeval.mp hx).comp ?_
75-
rw [← linearIndependent_iff_injective_linearCombination]
75+
rw [← linearIndependent_iff_injective_finsuppLinearCombination]
7676
exact linearIndependent_X _ _
7777

7878
protected theorem injective [Nontrivial R] : Injective x :=

0 commit comments

Comments
 (0)