Skip to content

Commit

Permalink
chore(DedekindDomain): drop a DecidableEq assumption (#11532)
Browse files Browse the repository at this point in the history
  • Loading branch information
urkud committed Mar 21, 2024
1 parent ebbc0fe commit b4f1310
Showing 1 changed file with 1 addition and 2 deletions.
3 changes: 1 addition & 2 deletions Mathlib/RingTheory/DedekindDomain/Ideal.lean
Expand Up @@ -712,8 +712,7 @@ theorem Ideal.prime_generator_of_prime {P : Ideal A} (h : Prime P) [P.IsPrincipa
prime_generator_of_isPrime _ h.ne_zero

open UniqueFactorizationMonoid in
nonrec theorem Ideal.mem_normalizedFactors_iff [DecidableEq (Ideal A)]
{p I : Ideal A} (hI : I ≠ ⊥) :
nonrec theorem Ideal.mem_normalizedFactors_iff {p I : Ideal A} (hI : I ≠ ⊥) :
p ∈ normalizedFactors I ↔ p.IsPrime ∧ I ≤ p := by
rw [← Ideal.dvd_iff_le]
by_cases hp : p = 0
Expand Down

0 comments on commit b4f1310

Please sign in to comment.