We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
gcd_eq_left
1 parent 88ab450 commit a3b56a9Copy full SHA for a3b56a9
Mathlib/Data/PNat/Prime.lean
@@ -253,12 +253,7 @@ theorem Coprime.gcd_mul (k : ℕ+) {m n : ℕ+} (h : m.Coprime n) :
253
rw [← coprime_coe] at h; apply eq
254
simp only [gcd_coe, mul_coe]; apply Nat.Coprime.gcd_mul k h
255
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
+@[deprecated (since := "2025-11-14")] alias ⟨_, gcd_eq_left⟩ := gcd_eq_left_iff_dvd
262
263
theorem Coprime.pow {m n : ℕ+} (k l : ℕ) (h : m.Coprime n) : (m ^ k : ℕ).Coprime (n ^ l) := by
264
rw [← coprime_coe] at *; apply Nat.Coprime.pow; apply h
0 commit comments