comm_alg/CommAlg/jayden(krull-dim-zero).lean

80 lines
2.4 KiB
Text
Raw Normal View History

2023-06-11 23:41:21 -05:00
import Mathlib.RingTheory.Ideal.Basic
2023-06-12 16:14:39 -05:00
import Mathlib.RingTheory.JacobsonIdeal
2023-06-11 23:41:21 -05:00
import Mathlib.RingTheory.Noetherian
2023-06-12 12:13:44 -05:00
import Mathlib.Order.KrullDimension
2023-06-11 23:41:21 -05:00
import Mathlib.RingTheory.Artinian
import Mathlib.RingTheory.Ideal.Quotient
import Mathlib.AlgebraicGeometry.PrimeSpectrum.Basic
2023-06-12 16:14:39 -05:00
import Mathlib.AlgebraicGeometry.PrimeSpectrum.Maximal
import Mathlib.Data.Finite.Defs
2023-06-11 23:41:21 -05:00
2023-06-12 16:14:39 -05:00
import Mathlib.Order.Height
import Mathlib.RingTheory.DedekindDomain.Basic
import Mathlib.RingTheory.Localization.AtPrime
import Mathlib.Order.ConditionallyCompleteLattice.Basic
2023-06-11 23:41:21 -05:00
2023-06-12 16:14:39 -05:00
-- copy from krull.lean; the name of Krull dimension for rings is changed to krullDim' since krullDim already exists in the librrary
namespace Ideal
2023-06-12 12:13:44 -05:00
2023-06-12 16:14:39 -05:00
variable (R : Type _) [CommRing R] (I : PrimeSpectrum R)
2023-06-12 12:13:44 -05:00
2023-06-12 16:14:39 -05:00
noncomputable def height : ℕ∞ := Set.chainHeight {J : PrimeSpectrum R | J < I}
noncomputable def krullDim' (R : Type) [CommRing R] : WithBot ℕ∞ := ⨆ (I : PrimeSpectrum R), height R I
-- copy ends
-- Stacks Lemma 10.60.5: R is Artinian iff R is Noetherian of dimension 0
2023-06-12 12:13:44 -05:00
lemma dim_zero_Noetherian_iff_Artinian (R : Type _) [CommRing R] :
2023-06-12 16:14:39 -05:00
IsNoetherianRing R ∧ krullDim' R = 0 ↔ IsArtinianRing R := by
2023-06-12 16:32:20 -05:00
2023-06-12 12:13:44 -05:00
variable {R : Type _} [CommRing R]
2023-06-11 23:41:21 -05:00
2023-06-12 12:13:44 -05:00
-- Repeats the definition by Monalisa
noncomputable def length : krullDim (Submodule _ _)
-- The following is Stacks Lemma 10.60.5
lemma dim_zero_Noetherian_iff_Artinian (R : Type _) [CommRing R] :
IsNoetherianRing R ∧ krull_dim R = 0 ↔ IsArtinianRing R := by
2023-06-12 16:32:20 -05:00
2023-06-12 12:13:44 -05:00
sorry
#check IsNoetherianRing
2023-06-12 16:14:39 -05:00
#check krullDim
-- Repeats the definition of the length of a module by Monalisa
variable (M : Type _) [AddCommMonoid M] [Module R M]
noncomputable def length := krullDim (Submodule R M)
#check length
-- Stacks Lemma 10.53.6: R is Artinian iff R has finite length as an R-mod
2023-06-12 12:13:44 -05:00
lemma IsArtinian_iff_finite_length : IsArtinianRing R ↔ ∃ n : , length R R ≤ n := by sorry
2023-06-11 23:41:21 -05:00
2023-06-12 16:14:39 -05:00
-- Stacks Lemma 10.53.3: R is Artinian iff R has finitely many maximal ideals
lemma IsArtinian_iff_finite_max_ideal : IsArtinianRing R ↔ Finite (MaximalSpectrum R) := by sorry
-- Stacks Lemma 10.53.4: R Artinian => Jacobson ideal of R is nilpotent
lemma Jacobson_of_Artinian_is_nilpotent : Is
-- how to use namespace
2023-06-11 23:41:21 -05:00
2023-06-12 16:14:39 -05:00
namespace something
2023-06-11 23:41:21 -05:00
2023-06-12 16:14:39 -05:00
end something
2023-06-11 23:41:21 -05:00
2023-06-12 16:14:39 -05:00
open something
2023-06-11 23:41:21 -05:00
2023-06-12 16:32:20 -05:00
-- The following is Stacks Lemma 10.53.6
lemma IsArtinian_iff_finite_length : IsArtinianRing R ↔ ∃ n : , length R R ≤ n := by sorry
2023-06-11 23:41:21 -05:00