Documentation

Mathlib.AlgebraicGeometry.Cover.Directed

Locally directed covers #

A locally directed P-cover of a scheme X is a cover 𝒰 with an ordering on the indices and compatible transition maps 𝒰ᵢ ⟶ 𝒰ⱼ for i ≤ j such that every x : 𝒰ᵢ ×[X] 𝒰ⱼ comes from some 𝒰ₖ for a k ≤ i and k ≤ j.

Gluing along directed covers is easier, because the intersections 𝒰ᵢ ×[X] 𝒰ⱼ can be covered by a subcover of 𝒰. In particular, if 𝒰 is a Zariski cover, X naturally is the colimit of the 𝒰ᵢ.

Many natural covers are naturally directed, most importantly the cover of all affine opens of a scheme.

A directed P-cover of a scheme X is a cover 𝒰 with an ordering on the indices and compatible transition maps 𝒰ᵢ ⟶ 𝒰ⱼ for i ≤ j such that every x : 𝒰ᵢ ×[X] 𝒰ⱼ comes from some 𝒰ₖ for a k ≤ i and k ≤ j.

Instances

    The transition maps of a directed cover.

    Equations
    Instances For
      theorem AlgebraicGeometry.Scheme.Cover.exists_lift_trans_eq {P : CategoryTheory.MorphismProperty Scheme} {X : Scheme} (𝒰 : Cover (precoverage P) X) [CategoryTheory.Category.{u_2, u_1} 𝒰.I₀] [𝒰.LocallyDirected] {i j : 𝒰.I₀} (x : (CategoryTheory.Limits.pullback (𝒰.f i) (𝒰.f j))) :
      ∃ (k : 𝒰.I₀) (hki : k i) (hkj : k j) (y : (𝒰.X k)), (CategoryTheory.ConcreteCategory.hom (CategoryTheory.Limits.pullback.lift (𝒰.trans hki) (𝒰.trans hkj) ).base) y = x

      If 𝒰 is a directed cover of X, this is the cover of 𝒰ᵢ ×[X] 𝒰ⱼ by {𝒰ₖ} where k ≤ i and k ≤ j.

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

        The canonical diagram induced by a locally directed cover.

        Equations
        Instances For

          The canonical cocone with point X on the functor induced by the locally directed cover 𝒰. If 𝒰 is an open cover, this is colimiting (see OpenCover.isColimitCoconeOfLocallyDirected).

          Equations
          Instances For
            def AlgebraicGeometry.Scheme.OpenCover.glueMorphismsOfLocallyDirected {X : Scheme} (𝒰 : X.OpenCover) [CategoryTheory.Category.{u_2, u_1} 𝒰.I₀] [Cover.LocallyDirected 𝒰] {Y : Scheme} (g : (i : 𝒰.I₀) → 𝒰.X i Y) (h : ∀ {i j : 𝒰.I₀} (hij : i j), CategoryTheory.CategoryStruct.comp (Cover.trans 𝒰 hij) (g j) = g i) :
            X Y

            If 𝒰 is a directed open cover of X, to glue morphisms {gᵢ : 𝒰ᵢ ⟶ Y} it suffices to check compatibility with the transition maps. See OpenCover.isColimitCoconeOfLocallyDirected for this result stated in the language of colimits.

            Equations
            Instances For
              @[simp]
              theorem AlgebraicGeometry.Scheme.OpenCover.map_glueMorphismsOfLocallyDirected {X : Scheme} (𝒰 : X.OpenCover) [CategoryTheory.Category.{u_2, u_1} 𝒰.I₀] [Cover.LocallyDirected 𝒰] {Y : Scheme} (g : (i : 𝒰.I₀) → 𝒰.X i Y) (h : ∀ {i j : 𝒰.I₀} (hij : i j), CategoryTheory.CategoryStruct.comp (Cover.trans 𝒰 hij) (g j) = g i) (i : 𝒰.I₀) :

              If 𝒰 is an open cover of X that is locally directed, X is the colimit of the components of 𝒰.

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

                If 𝒰 is a directed open cover of X, to glue morphisms {gᵢ : 𝒰ᵢ ⟶ Y} over S it suffices to check compatibility with the transition maps.

                Equations
                Instances For

                  If 𝒰 is an open cover such that the images of the components form a basis of the topology of X, 𝒰 is directed by the ordering of subset inclusion of the images.

                  Equations
                  • One or more equations did not get rendered due to their size.
                  Instances For
                    theorem AlgebraicGeometry.Scheme.Cover.LocallyDirected.ofIsBasisOpensRange_le_iff {X : Scheme} {𝒰 : X.OpenCover} [Preorder 𝒰.I₀] (hle : ∀ {i j : 𝒰.I₀}, i j Hom.opensRange (𝒰.f i) Hom.opensRange (𝒰.f j)) (i j : 𝒰.I₀) :
                    i j Hom.opensRange (𝒰.f i) Hom.opensRange (𝒰.f j)
                    theorem AlgebraicGeometry.Scheme.Cover.LocallyDirected.ofIsBasisOpensRange_trans {X : Scheme} {𝒰 : X.OpenCover} [Preorder 𝒰.I₀] (hle : ∀ {i j : 𝒰.I₀}, i j Hom.opensRange (𝒰.f i) Hom.opensRange (𝒰.f j)) (H : TopologicalSpace.Opens.IsBasis (Set.range fun (i : 𝒰.I₀) => Hom.opensRange (𝒰.f i))) {i j : 𝒰.I₀} (hij : i j) :
                    Cover.trans 𝒰 (CategoryTheory.homOfLE hij) = IsOpenImmersion.lift (𝒰.f j) (𝒰.f i)

                    The directed affine open cover of X given by all affine opens.

                    Equations
                    Instances For