Skip to content

Commit a3b56a9

Browse files
committed
chore(Data/PNat): deprecate gcd_eq_left (#31606)
1 parent 88ab450 commit a3b56a9

File tree

1 file changed

+1
-6
lines changed

1 file changed

+1
-6
lines changed

Mathlib/Data/PNat/Prime.lean

Lines changed: 1 addition & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -253,12 +253,7 @@ theorem Coprime.gcd_mul (k : ℕ+) {m n : ℕ+} (h : m.Coprime n) :
253253
rw [← coprime_coe] at h; apply eq
254254
simp only [gcd_coe, mul_coe]; apply Nat.Coprime.gcd_mul k h
255255

256-
theorem gcd_eq_left {m n : ℕ+} : m ∣ n → m.gcd n = m := by
257-
rw [dvd_iff]
258-
intro h
259-
apply eq
260-
simp only [gcd_coe]
261-
apply Nat.gcd_eq_left h
256+
@[deprecated (since := "2025-11-14")] alias ⟨_, gcd_eq_left⟩ := gcd_eq_left_iff_dvd
262257

263258
theorem Coprime.pow {m n : ℕ+} (k l : ℕ) (h : m.Coprime n) : (m ^ k : ℕ).Coprime (n ^ l) := by
264259
rw [← coprime_coe] at *; apply Nat.Coprime.pow; apply h

0 commit comments

Comments
 (0)