Skip to content

Commit 01fc25a

Browse files
committed
chore(Algebra/Bilinear): deprecate duplicated injectivity lemmas (#19231)
These are less general versions of results stated elsewhere. This partially deprecates @Vierkantor's leanprover-community/mathlib3#6588. Also tidy the one caller of these lemmas.
1 parent 08c6918 commit 01fc25a

File tree

2 files changed

+12
-15
lines changed

2 files changed

+12
-15
lines changed

Mathlib/Algebra/Algebra/Bilinear.lean

Lines changed: 10 additions & 13 deletions
Original file line numberDiff line numberDiff line change
@@ -225,22 +225,19 @@ section Ring
225225

226226
variable {R A : Type*} [CommSemiring R] [Ring A] [Algebra R A]
227227

228+
@[deprecated mul_right_injective₀ (since := "2024-11-18")]
228229
theorem mulLeft_injective [NoZeroDivisors A] {x : A} (hx : x ≠ 0) :
229-
Function.Injective (mulLeft R x) := by
230-
letI : Nontrivial A := ⟨⟨x, 0, hx⟩⟩
231-
letI := NoZeroDivisors.to_isDomain A
232-
exact mul_right_injective₀ hx
230+
Function.Injective (mulLeft R x) :=
231+
mul_right_injective₀ hx
233232

233+
@[deprecated mul_left_injective₀ (since := "2024-11-18")]
234234
theorem mulRight_injective [NoZeroDivisors A] {x : A} (hx : x ≠ 0) :
235-
Function.Injective (mulRight R x) := by
236-
letI : Nontrivial A := ⟨⟨x, 0, hx⟩⟩
237-
letI := NoZeroDivisors.to_isDomain A
238-
exact mul_left_injective₀ hx
239-
240-
theorem mul_injective [NoZeroDivisors A] {x : A} (hx : x ≠ 0) : Function.Injective (mul R A x) := by
241-
letI : Nontrivial A := ⟨⟨x, 0, hx⟩⟩
242-
letI := NoZeroDivisors.to_isDomain A
243-
exact mul_right_injective₀ hx
235+
Function.Injective (mulRight R x) :=
236+
mul_left_injective₀ hx
237+
238+
@[deprecated mul_right_injective₀ (since := "2024-11-18")]
239+
theorem mul_injective [NoZeroDivisors A] {x : A} (hx : x ≠ 0) : Function.Injective (mul R A x) :=
240+
mul_right_injective₀ hx
244241

245242
end Ring
246243

Mathlib/RingTheory/Ideal/Basis.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -21,7 +21,7 @@ variable {ι R S : Type*} [CommSemiring R] [CommRing S] [IsDomain S] [Algebra R
2121
noncomputable def basisSpanSingleton (b : Basis ι R S) {x : S} (hx : x ≠ 0) :
2222
Basis ι R (span ({x} : Set S)) :=
2323
b.map <|
24-
LinearEquiv.ofInjective (Algebra.lmul R S x) (LinearMap.mul_injective hx) ≪≫ₗ
24+
LinearEquiv.ofInjective (LinearMap.mulLeft R x) (mul_right_injective₀ hx) ≪≫ₗ
2525
LinearEquiv.ofEq _ _
2626
(by
2727
ext
@@ -33,7 +33,7 @@ theorem basisSpanSingleton_apply (b : Basis ι R S) {x : S} (hx : x ≠ 0) (i :
3333
(basisSpanSingleton b hx i : S) = x * b i := by
3434
simp only [basisSpanSingleton, Basis.map_apply, LinearEquiv.trans_apply,
3535
Submodule.restrictScalarsEquiv_apply, LinearEquiv.ofInjective_apply, LinearEquiv.coe_ofEq_apply,
36-
LinearEquiv.restrictScalars_apply, Algebra.coe_lmul_eq_mul, LinearMap.mul_apply']
36+
LinearEquiv.restrictScalars_apply, LinearMap.mulLeft_apply, LinearMap.mul_apply']
3737

3838
@[simp]
3939
theorem constr_basisSpanSingleton {N : Type*} [Semiring N] [Module N S] [SMulCommClass R N S]

0 commit comments

Comments
 (0)