comm_alg/CommAlg/sameer(artinian-rings).lean

16 lines
571 B
Text
Raw Normal View History

2023-06-12 12:34:51 -05:00
import Mathlib.RingTheory.Ideal.Basic
import Mathlib.RingTheory.Noetherian
import Mathlib.RingTheory.Artinian
import Mathlib.RingTheory.Ideal.Quotient
import Mathlib.AlgebraicGeometry.PrimeSpectrum.Basic
2023-06-12 15:34:09 -05:00
lemma quotientRing_is_Artinian (R : Type _) [CommRing R] (I : Ideal R) (IsArt : IsArtinianRing R):
IsArtinianRing (RI) := by sorry
#check Ideal.IsPrime
lemma IsPrimeMaximal (R : Type _) [CommRing R] (I : Ideal R) (IsArt : IsArtinianRing R) (isPrime : Ideal.IsPrime I) : Ideal.IsMaximal I := by sorry
2023-06-12 12:34:51 -05:00
-- Use Stacks project proof since it's broken into lemmas