added preliminary def of krullDimGE

This commit is contained in:
GTBarkley 2023-06-11 12:33:18 +00:00
parent e65513322c
commit dc034c2b09

View file

@ -37,3 +37,6 @@ lemma twoHeights : s ≠ ∅ → (some (Set.chainHeight s) : WithBot (WithTop
sorry
-- norm_cast
sorry
def krullDimGE (R : Type _) [CommRing R] (n : ) :=
∃ c : List (PrimeSpectrum R), c.Chain' (· < ·) ∧ c.length = n + 1