Documentation

Mathlib.AlgebraicGeometry.Sites.MorphismProperty

Site defined by a morphism property #

Given a multiplicative morphism property P that is stable under base change, we define the associated precoverage on the category of schemes, where coverings are given by jointly surjective families of morphisms satisfying P.

A morphism property of schemes is said to preserve joint surjectivity, if for any pair of morphisms f : X ⟶ S and g : Y ⟶ S where g satisfies P, any pair of points x : X and y : Y with f x = g y can be lifted to a point of X ×[S] Y.

In later files, this will be automatic, since this holds for any morphism g (see AlgebraicGeometry.Scheme.isJointlySurjectivePreserving). But at this early stage in the import tree, we only know it for open immersions.

Instances

    The precoverage on Scheme induced by P is given by jointly surjective families of P-morphisms.

    Equations
    Instances For
      @[simp]
      theorem AlgebraicGeometry.Scheme.ofArrows_mem_precoverage_iff (P : CategoryTheory.MorphismProperty Scheme) {S : Scheme} {ι : Type u_1} {X : ιScheme} {f : (i : ι) → X i S} :
      CategoryTheory.Presieve.ofArrows X f (precoverage P).coverings S (∀ (x : S), ∃ (i : ι), x Set.range (CategoryTheory.ConcreteCategory.hom (f i).base)) ∀ (i : ι), P (f i)
      @[reducible, inline]

      The Zariski precoverage on the category of schemes is the precoverage defined by jointly surjective families of open immersions.

      Equations
      Instances For