mirror of
https://github.com/GTBarkley/comm_alg.git
synced 2024-12-26 07:38:36 -06:00
changed type of 1 in dim_le_one_of_dimLEOne
This commit is contained in:
parent
50ec280145
commit
7173aefe8d
1 changed files with 2 additions and 1 deletions
|
@ -197,7 +197,8 @@ height 𝔭 > (n : WithBot ℕ∞) ↔ ∃ c : List (PrimeSpectrum R), c.Chain'
|
||||||
|
|
||||||
/-- The converse of this is false, because the definition of "dimension ≤ 1" in mathlib
|
/-- The converse of this is false, because the definition of "dimension ≤ 1" in mathlib
|
||||||
applies only to dimension zero rings and domains of dimension 1. -/
|
applies only to dimension zero rings and domains of dimension 1. -/
|
||||||
lemma dim_le_one_of_dimLEOne : Ring.DimensionLEOne R → krullDim R ≤ (1 : ℕ) := by
|
lemma dim_le_one_of_dimLEOne : Ring.DimensionLEOne R → krullDim R ≤ 1 := by
|
||||||
|
show _ → ((_ : WithBot ℕ∞) ≤ (1 : ℕ))
|
||||||
rw [krullDim_le_iff R 1]
|
rw [krullDim_le_iff R 1]
|
||||||
intro H p
|
intro H p
|
||||||
apply le_of_not_gt
|
apply le_of_not_gt
|
||||||
|
|
Loading…
Reference in a new issue