Documentation

Mathlib.RingTheory.Noetherian.OfPrime

Noetherian rings and prime ideals #

Main results #

References #

theorem Ideal.isOka_fg {R : Type u_1} [CommRing R] :

Ideal.FG is an Oka predicate.

theorem IsNoetherianRing.of_prime {R : Type u_1} [CommRing R] (H : ∀ (I : Ideal R), I.IsPrimeI.FG) :

If all prime ideals in a commutative ring are finitely generated, so are all other ideals.