File tree Expand file tree Collapse file tree 2 files changed +18
-0
lines changed
Mathlib/AlgebraicGeometry Expand file tree Collapse file tree 2 files changed +18
-0
lines changed Original file line number Diff line number Diff line change @@ -457,6 +457,17 @@ lemma isIntegralHom_over_iff_isEmpty : IsIntegralHom (𝔸(n; S) ↘ S) ↔ IsEm
457457lemma not_isIntegralHom [Nonempty S] [Nonempty n] : ¬ IsIntegralHom (𝔸(n; S) ↘ S) := by
458458 simp [isIntegralHom_over_iff_isEmpty]
459459
460+ lemma spec_le_iff (R : CommRingCat) (p q : Spec R) :
461+ p ≤ q ↔ q.asIdeal ≤ p.asIdeal := by aesop (add simp PrimeSpectrum.le_iff_specializes)
462+
463+ /--
464+ One should bear this equality in mind when breaking the `Spec R/ PrimeSpectrum R` abstraction
465+ boundary, since these instances are not definitionally equal.
466+ -/
467+ example (R : CommRingCat) :
468+ inferInstance (α := Preorder (Spec R)) =
469+ inferInstance (α := Preorder (PrimeSpectrum R)ᵒᵈ) := by aesop (add simp spec_le_iff)
470+
460471end instances
461472
462473end AffineSpace
Original file line number Diff line number Diff line change @@ -125,6 +125,13 @@ lemma Hom.continuous {X Y : Scheme} (f : X.Hom Y) : Continuous f.base := f.base.
125125protected abbrev sheaf (X : Scheme) :=
126126 X.toSheafedSpace.sheaf
127127
128+ /--
129+ We give schemes the specialization preorder by default.
130+ -/
131+ instance {X : Scheme.{u}} : Preorder X := specializationPreorder X
132+
133+ lemma le_iff_specializes {X : Scheme.{u}} {a b : X} : a ≤ b ↔ b ⤳ a := by rfl
134+
128135namespace Hom
129136
130137variable {X Y : Scheme.{u}} (f : Hom X Y) {U U' : Y.Opens} {V V' : X.Opens}
You can’t perform that action at this time.
0 commit comments