renamed comm_alg folder so imports work

This commit is contained in:
GTBarkley 2023-06-12 17:44:27 +00:00
parent 45c58bf041
commit c5a522392c
5 changed files with 15 additions and 22 deletions

View file

@ -2,6 +2,7 @@ import Mathlib.Order.KrullDimension
import Mathlib.Order.JordanHolder
import Mathlib.AlgebraicGeometry.PrimeSpectrum.Basic
import Mathlib.Order.Height
import CommAlg.krull
#check (p q : PrimeSpectrum _) → (p ≤ q)
@ -10,6 +11,9 @@ import Mathlib.Order.Height
-- Dimension of a ring
#check krullDim (PrimeSpectrum _)
#check Set.chainHeight {M' : Submodule _ _ | M' < _}
-- Length of a module
#check krullDim (Submodule _ _)
@ -39,22 +43,14 @@ lemma twoHeights : s ≠ ∅ → (some (Set.chainHeight s) : WithBot (WithTop
-- norm_cast
sorry
namespace Ideal
noncomputable def krullDim (R : Type _) [CommRing R] :=
Set.chainHeight (Set.univ : Set (PrimeSpectrum R))
def krullDimGE (R : Type _) [CommRing R] (n : ) :=
∃ c : List (PrimeSpectrum R), c.Chain' (· < ·) ∧ c.length = n + 1
def krullDimLE (R : Type _) [CommRing R] (n : ) :=
∀ c : List (PrimeSpectrum R), c.Chain' (· < ·) → c.length ≤ n + 1
end Ideal
open Ideal
lemma krullDim_le (R : Type _) [CommRing R] : krullDimLE R n ↔ Ideal.krullDim R ≤ n := sorry
lemma krullDim_ge (R : Type _) [CommRing R] : krullDimGE R n ↔ Ideal.krullDim R ≥ n := sorry
lemma krullDim_le_iff' (R : Type _) [CommRing R] :
Ideal.krullDim R ≤ n ↔ (∀ c : List (PrimeSpectrum R), c.Chain' (· < ·) → c.length ≤ n + 1) := by
sorry
lemma krullDim_ge_iff' (R : Type _) [CommRing R] :
Ideal.krullDim R ≥ n ↔ ∃ c : List (PrimeSpectrum R), c.Chain' (· < ·) ∧ c.length = n + 1 := sorry
-- #check ((4 : ℕ∞) : WithBot (WithTop ))

View file

@ -1,14 +1,11 @@
import Lake
open Lake DSL
package «comm_alg» {
-- add any package configuration options here
}
package comm_alg
@[default_target]
lean_lib CommAlg where
moreLeanArgs := #["-Dpp.unicode.fun=true"] -- pretty-prints `fun a ↦ b`
require mathlib from git
"https://github.com/leanprover-community/mathlib4.git"
@[default_target]
lean_lib «CommAlg» {
-- add any library configuration options here
}