File tree Expand file tree Collapse file tree 1 file changed +4
-1
lines changed
Mathlib/Algebra/Order/Group/Unbundled Expand file tree Collapse file tree 1 file changed +4
-1
lines changed Original file line number Diff line number Diff line change @@ -123,9 +123,12 @@ theorem abs_ediv_le_abs : ∀ a b : ℤ, |a / b| ≤ |a| :=
123
123
| -[m+1 ], 0 => Nat.zero_le _
124
124
| -[m+1 ], n + 1 => Nat.succ_le_succ (Nat.div_le_self _ _))
125
125
126
- theorem abs_sign_of_nonzero {z : ℤ} (hz : z ≠ 0 ) : |z.sign| = 1 := by
126
+ theorem abs_sign_of_ne_zero {z : ℤ} (hz : z ≠ 0 ) : |z.sign| = 1 := by
127
127
rw [abs_eq_natAbs, natAbs_sign_of_ne_zero hz, Int.ofNat_one]
128
128
129
+ @[deprecated (since := "2025-09-03")]
130
+ alias abs_sign_of_nonzero := abs_sign_of_ne_zero
131
+
129
132
protected theorem sign_eq_ediv_abs' (a : ℤ) : sign a = a / |a| :=
130
133
if az : a = 0 then by simp [az]
131
134
else (Int.ediv_eq_of_eq_mul_left (mt abs_eq_zero.1 az) (sign_mul_abs _).symm).symm
You can’t perform that action at this time.
0 commit comments