@@ -225,22 +225,19 @@ section Ring
225
225
226
226
variable {R A : Type *} [CommSemiring R] [Ring A] [Algebra R A]
227
227
228
+ @[deprecated mul_right_injective₀ (since := "2024-11-18")]
228
229
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
233
232
233
+ @[deprecated mul_left_injective₀ (since := "2024-11-18")]
234
234
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
244
241
245
242
end Ring
246
243
0 commit comments