Documentation

Mathlib.AlgebraicGeometry.Morphisms.Affine

Affine morphisms of schemes #

A morphism of schemes f : X ⟶ Y is affine if the preimage of an arbitrary affine open subset of Y is affine.

It is equivalent to ask only that Y is covered by affine opens whose preimage is affine.

Main results #

We also provide the instance HasAffineProperty @IsAffineHom fun X _ _ _ ↦ IsAffine X.

TODO #

A morphism of schemes X ⟶ Y is affine if the preimage of any affine open subset of Y is affine.

Instances
    def AlgebraicGeometry.affinePreimage {X : AlgebraicGeometry.Scheme} {Y : AlgebraicGeometry.Scheme} (f : X Y) [AlgebraicGeometry.IsAffineHom f] (U : Y.affineOpens) :
    X.affineOpens

    The preimage of an affine open as an Scheme.affine_opens.

    Equations
    Instances For
      Equations
      • =
      theorem AlgebraicGeometry.isAffineOpen_of_isAffineOpen_basicOpen_aux {X : AlgebraicGeometry.Scheme} (s : Set (X.presheaf.obj (Opposite.op ))) (hs : Ideal.span s = ) (hs₂ : is, AlgebraicGeometry.IsAffineOpen (X.basicOpen i)) :
      QuasiSeparatedSpace X.toPresheafedSpace
      theorem AlgebraicGeometry.isAffineOpen_of_isAffineOpen_basicOpen {X : AlgebraicGeometry.Scheme} (U : X.Opens) (s : Set (X.presheaf.obj (Opposite.op U))) (hs : Ideal.span s = ) (hs₂ : is, AlgebraicGeometry.IsAffineOpen (X.basicOpen i)) :

      If s is a spanning set of Γ(X, U), such that each X.basicOpen i is affine, then U is also affine.