Skip to content

Commit

Permalink
feat(AlgebraicGeometry): stability properties of separated (#17861)
Browse files Browse the repository at this point in the history
Separated is multiplicative, stable under base change and local at the target.
  • Loading branch information
chrisflav committed Oct 17, 2024
1 parent 035f251 commit d951eef
Showing 1 changed file with 18 additions and 3 deletions.
21 changes: 18 additions & 3 deletions Mathlib/AlgebraicGeometry/Morphisms/Separated.lean
Original file line number Diff line number Diff line change
Expand Up @@ -16,9 +16,6 @@ A morphism of schemes is separated if its diagonal morphism is a closed immmersi
## TODO
- Show separated is stable under composition and base change (this is immediate if
we show that closed immersions are stable under base change).
- Show separated is local at the target.
- Show affine morphisms are separated.
-/
Expand Down Expand Up @@ -60,6 +57,24 @@ instance : MorphismProperty.RespectsIso @IsSeparated := by

instance (priority := 900) [IsSeparated f] : QuasiSeparated f where

instance stableUnderComposition : MorphismProperty.IsStableUnderComposition @IsSeparated := by
rw [isSeparated_eq_diagonal_isClosedImmersion]
exact MorphismProperty.diagonal_isStableUnderComposition IsClosedImmersion.stableUnderBaseChange

instance {Z : Scheme.{u}} (g : Y ⟶ Z) [IsSeparated f] [IsSeparated g] : IsSeparated (f ≫ g) :=
stableUnderComposition.comp_mem f g inferInstance inferInstance

instance : MorphismProperty.IsMultiplicative @IsSeparated where
id_mem _ := inferInstance

lemma stableUnderBaseChange : MorphismProperty.StableUnderBaseChange @IsSeparated := by
rw [isSeparated_eq_diagonal_isClosedImmersion]
exact MorphismProperty.StableUnderBaseChange.diagonal IsClosedImmersion.stableUnderBaseChange

instance : IsLocalAtTarget @IsSeparated := by
rw [isSeparated_eq_diagonal_isClosedImmersion]
infer_instance

end IsSeparated

end AlgebraicGeometry

0 comments on commit d951eef

Please sign in to comment.