Skip to content

Commit b9715de

Browse files
chore: remove duplicate prodPrimeFactors_apply_of_ne_zero (#9366)
1 parent 3694e27 commit b9715de

File tree

1 file changed

+1
-5
lines changed

1 file changed

+1
-5
lines changed

Mathlib/NumberTheory/ArithmeticFunction.lean

Lines changed: 1 addition & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -586,10 +586,6 @@ theorem prodPrimeFactors_apply [CommMonoidWithZero R] {f: ℕ → R} {n : ℕ} (
586586
∏ᵖ p ∣ n, f p = ∏ p in n.primeFactors, f p :=
587587
if_neg hn
588588

589-
theorem prodPrimeFactors_apply_of_ne_zero [CommMonoidWithZero R] {f : ℕ → R} {n : ℕ}
590-
(hn : n ≠ 0) : ∏ᵖ p ∣ n, f p = ∏ p in n.primeFactors, f p :=
591-
prodPrimeFactors_apply hn
592-
593589
end ProdPrimeFactors
594590

595591
/-- Multiplicative functions -/
@@ -775,7 +771,7 @@ theorem prodPrimeFactors [CommMonoidWithZero R] (f : ℕ → R) :
775771
theorem prodPrimeFactors_add_of_squarefree [CommSemiring R] {f g : ArithmeticFunction R}
776772
(hf : IsMultiplicative f) (hg : IsMultiplicative g) {n : ℕ} (hn : Squarefree n) :
777773
∏ᵖ p ∣ n, (f + g) p = (f * g) n := by
778-
rw [prodPrimeFactors_apply_of_ne_zero hn.ne_zero]
774+
rw [prodPrimeFactors_apply hn.ne_zero]
779775
simp_rw [add_apply (f:=f) (g:=g)]
780776
rw [Finset.prod_add, mul_apply, sum_divisorsAntidiagonal (f · * g ·),
781777
← divisors_filter_squarefree_of_squarefree hn, sum_divisors_filter_squarefree hn.ne_zero,

0 commit comments

Comments
 (0)