Documentation

Mathlib.RingTheory.Ideal.MinimalPrime

Minimal primes #

We provide various results concerning the minimal primes above an ideal

Main results #

def Ideal.minimalPrimes {R : Type u_1} [CommRing R] (I : Ideal R) :

I.minimalPrimes is the set of ideals that are minimal primes over I.

Instances For
    def minimalPrimes (R : Type u_3) [CommRing R] :

    minimalPrimes R is the set of minimal primes of R. This is defined as Ideal.minimalPrimes.

    Instances For
      theorem Ideal.exists_minimalPrimes_le {R : Type u_1} [CommRing R] {I : Ideal R} {J : Ideal R} [Ideal.IsPrime J] (e : I J) :
      theorem Ideal.exists_comap_eq_of_mem_minimalPrimes_of_injective {R : Type u_1} {S : Type u_2} [CommRing R] [CommRing S] {f : R →+* S} (hf : Function.Injective f) (p : Ideal R) (H : p minimalPrimes R) :
      p', Ideal.IsPrime p' Ideal.comap f p' = p
      theorem Ideal.exists_comap_eq_of_mem_minimalPrimes {R : Type u_1} {S : Type u_2} [CommRing R] [CommRing S] {I : Ideal S} (f : R →+* S) (p : Ideal R) (H : p Ideal.minimalPrimes (Ideal.comap f I)) :
      p', Ideal.IsPrime p' I p' Ideal.comap f p' = p
      theorem Ideal.exists_minimalPrimes_comap_eq {R : Type u_1} {S : Type u_2} [CommRing R] [CommRing S] {I : Ideal S} (f : R →+* S) (p : Ideal R) (H : p Ideal.minimalPrimes (Ideal.comap f I)) :