Finitely generated ideals #
Lemmas about finiteness of ideal operations.
theorem
Ideal.fg_ker_comp
{R : Type u_3}
{S : Type u_4}
{A : Type u_5}
[CommRing R]
[CommRing S]
[CommRing A]
(f : R →+* S)
(g : S →+* A)
(hf : (RingHom.ker f).FG)
(hg : (RingHom.ker g).FG)
(hsur : Function.Surjective ⇑f)
:
(RingHom.ker (g.comp f)).FG
theorem
Ideal.exists_radical_pow_le_of_fg
{R : Type u_3}
[CommSemiring R]
(I : Ideal R)
(h : I.radical.FG)
:
theorem
Ideal.exists_pow_le_of_le_radical_of_fg_radical
{R : Type u_3}
[CommSemiring R]
{I J : Ideal R}
(hIJ : I ≤ J.radical)
(hJ : J.radical.FG)
:
@[deprecated Ideal.exists_pow_le_of_le_radical_of_fg_radical]
theorem
Ideal.exists_pow_le_of_le_radical_of_fG
{R : Type u_3}
[CommSemiring R]
{I J : Ideal R}
(hIJ : I ≤ J.radical)
(hJ : J.radical.FG)
:
theorem
Ideal.exists_pow_le_of_le_radical_of_fg
{R : Type u_3}
[CommSemiring R]
{I J : Ideal R}
(h' : I ≤ J.radical)
(h : I.FG)
: