Documentation

Mathlib.Topology.Sheaves.Stalks

Stalks #

For a presheaf F on a topological space X, valued in some category C, the stalk of F at the point x : X is defined as the colimit of the composition of the inclusion of categories (OpenNhds x)ᵒᵖ ⥤ (Opens X)ᵒᵖ and the functor F : (Opens X)ᵒᵖ ⥤ C. For an open neighborhood U of x, we define the map F.germ x : F.obj (op U) ⟶ F.stalk x as the canonical morphism into this colimit.

Taking stalks is functorial: For every point x : X we define a functor stalkFunctor C x, sending presheaves on X to objects of C. Furthermore, for a map f : X ⟶ Y between topological spaces, we define stalkPushforward as the induced map on the stalks (f _* ℱ).stalk (f x) ⟶ ℱ.stalk x.

Some lemmas about stalks and germs only hold for certain classes of concrete categories. A basic property of forgetful functors of categories of algebraic structures (like MonCat, CommRingCat,...) is that they preserve filtered colimits. Since stalks are filtered colimits, this ensures that the stalks of presheaves valued in these categories behave exactly as for Type-valued presheaves. For example, in germ_exist we prove that in such a category, every element of the stalk is the germ of a section.

Furthermore, if we require the forgetful functor to reflect isomorphisms and preserve limits (as is the case for most algebraic structures), we have access to the unique gluing API and can prove further properties. Most notably, in is_iso_iff_stalk_functor_map_iso, we prove that in such a category, a morphism of sheaves is an isomorphism if and only if all of its stalk maps are isomorphisms.

See also the definition of "algebraic structures" in the stacks project: https://stacks.math.columbia.edu/tag/007L

Stalks are functorial with respect to morphisms of presheaves over a fixed X.

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

    The stalk of a presheaf F at a point x is calculated as the colimit of the functor nbhds x ⥤ opens F.X ⥤ C

    Equations
    Instances For

      The germ of a section of a presheaf over an open at a point of that open.

      Equations
      Instances For
        theorem TopCat.Presheaf.germ_res {C : Type u} [CategoryTheory.Category.{v, u} C] [CategoryTheory.Limits.HasColimits C] {X : TopCat} (F : TopCat.Presheaf C X) {U : TopologicalSpace.Opens X} {V : TopologicalSpace.Opens X} (i : U V) (x : U) :
        CategoryTheory.CategoryStruct.comp (F.map i.op) (TopCat.Presheaf.germ F x) = TopCat.Presheaf.germ F ((fun (x : U) => { val := x, property := }) x)
        theorem TopCat.Presheaf.germ_res_apply {C : Type u} [CategoryTheory.Category.{v, u} C] [CategoryTheory.Limits.HasColimits C] {X : TopCat} (F : TopCat.Presheaf C X) {U : TopologicalSpace.Opens X} {V : TopologicalSpace.Opens X} (i : U V) (x : U) [CategoryTheory.ConcreteCategory C] (s : (CategoryTheory.forget C).obj (F.obj (Opposite.op V))) :
        (TopCat.Presheaf.germ F x) ((F.map i.op) s) = (TopCat.Presheaf.germ F ((fun (x : U) => { val := x, property := }) x)) s
        theorem TopCat.Presheaf.stalk_hom_ext {C : Type u} [CategoryTheory.Category.{v, u} C] [CategoryTheory.Limits.HasColimits C] {X : TopCat} (F : TopCat.Presheaf C X) {x : X} {Y : C} {f₁ : TopCat.Presheaf.stalk F x Y} {f₂ : TopCat.Presheaf.stalk F x Y} (ih : ∀ (U : TopologicalSpace.Opens X) (hxU : x U), CategoryTheory.CategoryStruct.comp (TopCat.Presheaf.germ F { val := x, property := hxU }) f₁ = CategoryTheory.CategoryStruct.comp (TopCat.Presheaf.germ F { val := x, property := hxU }) f₂) :
        f₁ = f₂

        A morphism from the stalk of F at x to some object Y is completely determined by its composition with the germ morphisms.

        For a presheaf F on a space X, a continuous map f : X ⟶ Y induces a morphisms between the stalk of f _ * F at f x and the stalk of F at x.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          @[simp]
          theorem TopCat.Presheaf.stalkPushforward_germ_apply (C : Type u) [CategoryTheory.Category.{v, u} C] [CategoryTheory.Limits.HasColimits C] {X : TopCat} {Y : TopCat} (f : X Y) (F : TopCat.Presheaf C X) (U : TopologicalSpace.Opens Y) (x : ((TopologicalSpace.Opens.map f).obj U)) [inst : CategoryTheory.ConcreteCategory C] (x : (CategoryTheory.forget C).obj ((f _* F).obj (Opposite.op U))) :
          (TopCat.Presheaf.stalkPushforward C f F x✝) ((TopCat.Presheaf.germ (f _* F) { val := f x✝, property := }) x) = (TopCat.Presheaf.germ F x✝) x

          The morphism ℱ_{f x} ⟶ (f⁻¹ℱ)ₓ that factors through (f_*f⁻¹ℱ)_{f x}.

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

            The morphism (f⁻¹ℱ)(U) ⟶ ℱ_{f(x)} for some U ∋ x.

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

              The morphism (f⁻¹ℱ)ₓ ⟶ ℱ_{f(x)}.

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

                The isomorphism ℱ_{f(x)} ≅ (f⁻¹ℱ)ₓ.

                Equations
                Instances For

                  If x specializes to y, then there is a natural map F.stalk y ⟶ F.stalk x.

                  Equations
                  • One or more equations did not get rendered due to their size.
                  Instances For
                    theorem TopCat.Presheaf.germ_stalkSpecializes' {C : Type u} [CategoryTheory.Category.{v, u} C] [CategoryTheory.Limits.HasColimits C] {X : TopCat} (F : TopCat.Presheaf C X) {U : TopologicalSpace.Opens X} {x : X} {y : X} (h : x y) (hy : y U) :
                    CategoryTheory.CategoryStruct.comp (TopCat.Presheaf.germ F { val := y, property := hy }) (TopCat.Presheaf.stalkSpecializes F h) = TopCat.Presheaf.germ F { val := x, property := }

                    The stalks are isomorphic on inseparable points

                    Equations
                    Instances For
                      theorem TopCat.Presheaf.germ_ext {C : Type u} [CategoryTheory.Category.{v, u} C] [CategoryTheory.Limits.HasColimits C] {X : TopCat} [CategoryTheory.ConcreteCategory C] (F : TopCat.Presheaf C X) {U : TopologicalSpace.Opens X} {V : TopologicalSpace.Opens X} {x : X} {hxU : x U} {hxV : x V} (W : TopologicalSpace.Opens X) (hxW : x W) (iWU : W U) (iWV : W V) {sU : (CategoryTheory.forget C).obj (F.obj (Opposite.op U))} {sV : (CategoryTheory.forget C).obj (F.obj (Opposite.op V))} (ih : (F.map iWU.op) sU = (F.map iWV.op) sV) :
                      (TopCat.Presheaf.germ F { val := x, property := hxU }) sU = (TopCat.Presheaf.germ F { val := x, property := hxV }) sV

                      For presheaves valued in a concrete category whose forgetful functor preserves filtered colimits, every element of the stalk is the germ of a section.

                      theorem TopCat.Presheaf.germ_eq {C : Type u} [CategoryTheory.Category.{v, u} C] [CategoryTheory.Limits.HasColimits C] {X : TopCat} [CategoryTheory.ConcreteCategory C] [CategoryTheory.Limits.PreservesFilteredColimits (CategoryTheory.forget C)] (F : TopCat.Presheaf C X) {U : TopologicalSpace.Opens X} {V : TopologicalSpace.Opens X} (x : X) (mU : x U) (mV : x V) (s : (CategoryTheory.forget C).obj (F.obj (Opposite.op U))) (t : (CategoryTheory.forget C).obj (F.obj (Opposite.op V))) (h : (TopCat.Presheaf.germ F { val := x, property := mU }) s = (TopCat.Presheaf.germ F { val := x, property := mV }) t) :
                      ∃ (W : TopologicalSpace.Opens X) (_ : x W) (iU : W U) (iV : W V), (F.map iU.op) s = (F.map iV.op) t

                      Let F be a sheaf valued in a concrete category, whose forgetful functor reflects isomorphisms, preserves limits and filtered colimits. Then two sections who agree on every stalk must be equal.

                      For surjectivity, we are given an arbitrary section t and need to find a preimage for it. We claim that it suffices to find preimages locally. That is, for each x : U we construct a neighborhood V ≤ U and a section s : F.obj (op V)) such that f.app (op V) s and t agree on V.

                      Let F and G be sheaves valued in a concrete category, whose forgetful functor reflects isomorphisms, preserves limits and filtered colimits. Then if the stalk maps of a morphism f : F ⟶ G are all isomorphisms, f must be an isomorphism.

                      Let F and G be sheaves valued in a concrete category, whose forgetful functor reflects isomorphisms, preserves limits and filtered colimits. Then a morphism f : F ⟶ G is an isomorphism if and only if all of its stalk maps are isomorphisms.