Skip to content

Commit e9d357f

Browse files
1 parent b26156e commit e9d357f

File tree

1 file changed

+4
-1
lines changed
  • Mathlib/Algebra/Order/Group/Unbundled

1 file changed

+4
-1
lines changed

Mathlib/Algebra/Order/Group/Unbundled/Int.lean

Lines changed: 4 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -123,9 +123,12 @@ theorem abs_ediv_le_abs : ∀ a b : ℤ, |a / b| ≤ |a| :=
123123
| -[m+1], 0 => Nat.zero_le _
124124
| -[m+1], n + 1 => Nat.succ_le_succ (Nat.div_le_self _ _))
125125

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
127127
rw [abs_eq_natAbs, natAbs_sign_of_ne_zero hz, Int.ofNat_one]
128128

129+
@[deprecated (since := "2025-09-03")]
130+
alias abs_sign_of_nonzero := abs_sign_of_ne_zero
131+
129132
protected theorem sign_eq_ediv_abs' (a : ℤ) : sign a = a / |a| :=
130133
if az : a = 0 then by simp [az]
131134
else (Int.ediv_eq_of_eq_mul_left (mt abs_eq_zero.1 az) (sign_mul_abs _).symm).symm

0 commit comments

Comments
 (0)