Skip to content

Commit

Permalink
fix
Browse files Browse the repository at this point in the history
  • Loading branch information
alreadydone committed Nov 20, 2024
1 parent 9104865 commit 2bbc76c
Show file tree
Hide file tree
Showing 2 changed files with 4 additions and 4 deletions.
2 changes: 1 addition & 1 deletion Mathlib/AlgebraicGeometry/PrimeSpectrum/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -226,7 +226,7 @@ theorem discreteTopology_iff_finite_isMaximal_and_sInf_le_nilradical :
letI s := {I : Ideal R | I.IsMaximal}
DiscreteTopology (PrimeSpectrum R) ↔ Finite s ∧ sInf s ≤ nilradical R :=
discreteTopology_iff_finite_and_isPrime_imp_isMaximal.trans <| by
simp_rw [(equivSetOfIsPrime R).finite_iff, Set.finite_coe_iff]
rw [(equivSetOfIsPrime R).finite_iff, ← Set.coe_setOf, Set.finite_coe_iff, Set.finite_coe_iff]
refine ⟨fun h ↦ ⟨h.1.subset fun _ h ↦ h.isPrime, nilradical_eq_sInf R ▸ sInf_le_sInf h.2⟩,
fun ⟨fin, le⟩ ↦ ?_⟩
have hpm (I : Ideal R) (hI : I.IsPrime): I.IsMaximal := by
Expand Down
6 changes: 3 additions & 3 deletions Mathlib/RingTheory/PrimeSpectrum.lean
Original file line number Diff line number Diff line change
Expand Up @@ -85,9 +85,9 @@ variable (R S)

/-- The prime spectrum is in bijection with the set of prime ideals. -/
@[simps]
def equivSetOfIsPrime : PrimeSpectrum R ≃ {I : Ideal R | I.IsPrime} where
toFun I := ⟨I.1, I.2
invFun I := ⟨I.1, I.2
def equivSetOfIsPrime : PrimeSpectrum R ≃ {I : Ideal R // I.IsPrime} where
toFun I := ⟨I.asIdeal, I.2
invFun I := ⟨I, I.2
left_inv _ := rfl
right_inv _ := rfl

Expand Down

0 comments on commit 2bbc76c

Please sign in to comment.