mathlib3 documentation

ring_theory.ideal.minimal_prime

Minimal primes #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

We provide various results concerning the minimal primes above an ideal

Main results #

def ideal.minimal_primes {R : Type u_1} [comm_ring R] (I : ideal R) :

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

Equations
def minimal_primes (R : Type u_1) [comm_ring R] :

minimal_primes R is the set of minimal primes of R. This is defined as ideal.minimal_primes.

Equations
theorem ideal.exists_minimal_primes_le {R : Type u_1} [comm_ring R] {I J : ideal R} [J.is_prime] (e : I J) :
(p : ideal R) (H : p I.minimal_primes), p J
@[simp]
theorem ideal.exists_comap_eq_of_mem_minimal_primes_of_injective {R : Type u_1} {S : Type u_2} [comm_ring R] [comm_ring S] {f : R →+* S} (hf : function.injective f) (p : ideal R) (H : p minimal_primes R) :
(p' : ideal S), p'.is_prime ideal.comap f p' = p
theorem ideal.exists_comap_eq_of_mem_minimal_primes {R : Type u_1} {S : Type u_2} [comm_ring R] [comm_ring S] {I : ideal S} (f : R →+* S) (p : ideal R) (H : p (ideal.comap f I).minimal_primes) :
(p' : ideal S), p'.is_prime I p' ideal.comap f p' = p
theorem ideal.exists_minimal_primes_comap_eq {R : Type u_1} {S : Type u_2} [comm_ring R] [comm_ring S] {I : ideal S} (f : R →+* S) (p : ideal R) (H : p (ideal.comap f I).minimal_primes) :
(p' : ideal S) (H : p' I.minimal_primes), ideal.comap f p' = p