Proper morphisms #
A morphism of schemes is proper if it is separated, universally closed and (locally) of finite type. Note that we don't require quasi-compact, since this is implied by universally closed (TODO).
class
AlgebraicGeometry.IsProper
{X Y : AlgebraicGeometry.Scheme}
(f : X ⟶ Y)
extends AlgebraicGeometry.IsSeparated f, AlgebraicGeometry.UniversallyClosed f, AlgebraicGeometry.LocallyOfFiniteType f :
A morphism is proper if it is separated, universally closed and locally of finite type.
- out : (AlgebraicGeometry.topologically @IsClosedMap).universally f
- finiteType_of_affine_subset : ∀ (U : ↑Y.affineOpens) (V : ↑X.affineOpens) (e : ↑V ≤ (TopologicalSpace.Opens.map f.base).obj ↑U), RingHom.FiniteType (AlgebraicGeometry.Scheme.Hom.appLE f (↑U) (↑V) e)
Instances
@[instance 900]
instance
AlgebraicGeometry.IsProper.instOfIsClosedImmersion
{X Y : AlgebraicGeometry.Scheme}
(f : X ⟶ Y)
[AlgebraicGeometry.IsClosedImmersion f]
:
Equations
- ⋯ = ⋯