Skip to content

Commit

Permalink
chore(RingTheory/Jacobson): Rename Ideal.IsJacobson to `IsJacobsonR…
Browse files Browse the repository at this point in the history
…ing`. (#18271)
  • Loading branch information
erdOne committed Oct 31, 2024
1 parent c169023 commit 2e82aa2
Show file tree
Hide file tree
Showing 3 changed files with 212 additions and 144 deletions.
8 changes: 4 additions & 4 deletions Mathlib/AlgebraicGeometry/PrimeSpectrum/Jacobson.lean
Original file line number Diff line number Diff line change
Expand Up @@ -22,11 +22,11 @@ import Mathlib.RingTheory.Jacobson

open Ideal

variable {R : Type*} [CommRing R] [IsJacobson R]
variable {R : Type*} [CommRing R] [IsJacobsonRing R]

namespace PrimeSpectrum

lemma exists_isClosed_singleton_of_isJacobson
lemma exists_isClosed_singleton_of_isJacobsonRing
(s : (Set (PrimeSpectrum R))) (hs : IsOpen s) (hs' : s.Nonempty) :
∃ x ∈ s, IsClosed {x} := by
simp_rw [isClosed_singleton_iff_isMaximal]
Expand All @@ -48,12 +48,12 @@ If `R` is both noetherian and jacobson, then the following are equivalent for `x
3. `{x}` is both closed and stable under generalization
(i.e. `x` is both a minimal prime and a maximal ideal)
-/
lemma isOpen_singleton_tfae_of_isNoetherian_of_isJacobson
lemma isOpen_singleton_tfae_of_isNoetherian_of_isJacobsonRing
[IsNoetherianRing R] (x : PrimeSpectrum R) :
List.TFAE [IsOpen {x}, IsClopen {x}, IsClosed {x} ∧ StableUnderGeneralization {x}] := by
tfae_have 12
· intro h
obtain ⟨y, rfl : y = x, h'⟩ := exists_isClosed_singleton_of_isJacobson _ h
obtain ⟨y, rfl : y = x, h'⟩ := exists_isClosed_singleton_of_isJacobsonRing _ h
⟨x, Set.mem_singleton x⟩
exact ⟨h', h⟩
tfae_have 23
Expand Down
Loading

0 comments on commit 2e82aa2

Please sign in to comment.