Documentation

Mathlib.RingTheory.UniqueFactorizationDomain.Ideal

Unique factorization and ascending chain condition on ideals #

Main results #

theorem Ideal.IsPrime.exists_mem_prime_of_ne_bot {R : Type u_2} [CommSemiring R] [IsDomain R] [UniqueFactorizationMonoid R] {I : Ideal R} (hI₂ : I.IsPrime) (hI : I ) :
xI, Prime x

Every non-zero prime ideal in a unique factorization domain contains a prime element.

theorem Ideal.setOf_isPrincipal_wellFoundedOn_gt {α : Type u_1} [CommSemiring α] [WfDvdMonoid α] [IsDomain α] :
{I : Ideal α | Submodule.IsPrincipal I}.WellFoundedOn fun (x1 x2 : Ideal α) => x1 > x2

The ascending chain condition on principal ideals holds in a WfDvdMonoid domain.

theorem WfDvdMonoid.of_setOf_isPrincipal_wellFoundedOn_gt {α : Type u_1} [CommSemiring α] [IsDomain α] (h : {I : Ideal α | Submodule.IsPrincipal I}.WellFoundedOn fun (x1 x2 : Ideal α) => x1 > x2) :

The ascending chain condition on principal ideals in a domain is sufficient to prove that the domain is WfDvdMonoid.