Documentation

Mathlib.AlgebraicGeometry.Sites.SmallAffineZariski

The small affine Zariski site #

X.AffineZariskiSite is the small affine Zariski site of X, whose elements are affine open sets of X, and whose arrows are basic open sets D(f) ⟶ U for any f : Γ(X, U).

Every presieve on U is then given by a Set Γ(X, U) (presieveOfSections_surjective), and we endow X.AffineZariskiSite with grothendieckTopology X, such that s : Set Γ(X, U) is a cover if and only if Ideal.span s = ⊤ (generate_presieveOfSections_mem_grothendieckTopology).

This is a dense subsite of X.Opens (with respect to Opens.grothendieckTopology X) via the inclusion functor toOpensFunctor X, which gives an equivalence of categories of sheaves (sheafEquiv).

Note that this differs from the definition on stacks project where the arrows in the small affine Zariski site are arbitrary inclusions.

X.AffineZariskiSite is the small affine Zariski site of X, whose elements are affine open sets of X, and whose arrows are basic open sets D(f) ⟶ U for any f : Γ(X, U).

Note that this differs from the definition on stacks project where the arrows in the small affine Zariski site are arbitrary inclusions.

Equations
Instances For
    @[reducible, inline]
    abbrev AlgebraicGeometry.Scheme.AffineZariskiSite.toOpens {X : Scheme} (U : X.AffineZariskiSite) :
    X.Opens

    The inclusion from X.AffineZariskiSite to X.Opens.

    Equations
    • U.toOpens = U
    Instances For
      def AlgebraicGeometry.Scheme.AffineZariskiSite.basicOpen {X : Scheme} (U : X.AffineZariskiSite) (f : (X.presheaf.obj (Opposite.op U.toOpens))) :
      X.AffineZariskiSite

      The basic open set of a section, as an element of AffineZariskiSite.

      Equations
      • U.basicOpen f = X.basicOpen f,
      Instances For
        theorem AlgebraicGeometry.Scheme.AffineZariskiSite.basicOpen_le {X : Scheme} (U : X.AffineZariskiSite) (f : (X.presheaf.obj (Opposite.op U.toOpens))) :
        U.basicOpen f U

        The inclusion functor from X.AffineZariskiSite to X.Opens.

        Equations
        Instances For

          The grothendieck topology on X.AffineZariskiSite induced from the topology on X.Opens. Also see mem_grothendieckTopology_iff_sectionsOfPresieve.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            theorem AlgebraicGeometry.Scheme.AffineZariskiSite.mem_grothendieckTopology {X : Scheme} {U : X.AffineZariskiSite} {S : CategoryTheory.Sieve U} :
            S (grothendieckTopology X) U xU.toOpens, ∃ (V : X.AffineZariskiSite) (f : V U), S.arrows f x V.toOpens
            def AlgebraicGeometry.Scheme.AffineZariskiSite.presieveOfSections {X : Scheme} (U : X.AffineZariskiSite) (s : Set (X.presheaf.obj (Opposite.op U.toOpens))) :

            The presieve associated to a set of sections. This is a surjection, see presieveOfSections_surjective.

            Equations
            • U.presieveOfSections s x✝ = fs, X.basicOpen f = V.toOpens
            Instances For
              def AlgebraicGeometry.Scheme.AffineZariskiSite.sectionsOfPresieve {X : Scheme} {U : X.AffineZariskiSite} (P : CategoryTheory.Presieve U) :
              Set (X.presheaf.obj (Opposite.op U.toOpens))

              The set of sections associated to a presieve.

              Equations
              Instances For
                theorem AlgebraicGeometry.Scheme.AffineZariskiSite.presieveOfSections_eq_ofArrows {X : Scheme} (U : X.AffineZariskiSite) (s : Set (X.presheaf.obj (Opposite.op U.toOpens))) :
                U.presieveOfSections s = CategoryTheory.Presieve.ofArrows (fun (i : s) => U.basicOpen i) fun (i : s) => CategoryTheory.homOfLE
                theorem AlgebraicGeometry.Scheme.AffineZariskiSite.generate_presieveOfSections {X : Scheme} {U V : X.AffineZariskiSite} {s : Set (X.presheaf.obj (Opposite.op U.toOpens))} {f : V U} :
                (CategoryTheory.Sieve.generate (U.presieveOfSections s)).arrows f fs, ∃ (g : (X.presheaf.obj (Opposite.op U.toOpens))), X.basicOpen (f * g) = V.toOpens
                @[reducible, inline]

                The category of sheaves on X.AffineZariskiSite is equivalent to the categories of sheaves over X.

                Equations
                • One or more equations did not get rendered due to their size.
                Instances For