Documentation

Mathlib.AlgebraicGeometry.LocallyRingedSpace

The category of locally ringed spaces #

We define (bundled) locally ringed spaces (as SheafedSpace CommRing along with the fact that the stalks are local rings), and morphisms between these (morphisms in SheafedSpace with is_local_ring_hom on the stalk maps).

A LocallyRingedSpace is a topological space equipped with a sheaf of commutative rings such that all the stalks are local rings.

A morphism of locally ringed spaces is a morphism of ringed spaces such that the morphisms induced on stalks are local ring homomorphisms.

Instances For

    An alias for to_SheafedSpace, where the result type is a RingedSpace. This allows us to use dot-notation for the RingedSpace namespace.

    Instances For

      The underlying topological space of a locally ringed space.

      Instances For

        A morphism of locally ringed spaces is a morphism of ringed spaces such that the morphisms induced on stalks are local ring homomorphisms.

        Instances For

          The stalk of a locally ringed space, just as a CommRing.

          Instances For

            A morphism of locally ringed spaces f : X ⟶ Y induces a local ring homomorphism from Y.stalk (f x) to X.stalk x for any x : X.

            Instances For

              Given two locally ringed spaces X and Y, an isomorphism between X and Y as sheafed spaces can be lifted to a morphism X ⟶ Y as locally ringed spaces.

              See also iso_of_SheafedSpace_iso.

              Instances For

                Given two locally ringed spaces X and Y, an isomorphism between X and Y as sheafed spaces can be lifted to an isomorphism X ⟶ Y as locally ringed spaces.

                This is related to the property that the functor forget_to_SheafedSpace reflects isomorphisms. In fact, it is slightly stronger as we do not require f to come from a morphism between locally ringed spaces.

                Instances For
                  @[simp]
                  theorem AlgebraicGeometry.LocallyRingedSpace.restrict_presheaf_map {U : TopCat} (X : AlgebraicGeometry.LocallyRingedSpace) {f : U AlgebraicGeometry.LocallyRingedSpace.toTopCat X} (h : OpenEmbedding f) :
                  ∀ {X Y : (TopologicalSpace.Opens U)ᵒᵖ} (f : X Y), (AlgebraicGeometry.LocallyRingedSpace.restrict X h).toSheafedSpace.toPresheafedSpace.presheaf.map f = X.presheaf.map ((IsOpenMap.functor (_ : IsOpenMap f)).map f.unop).op

                  The restriction of a locally ringed space X to the top subspace is isomorphic to X itself.

                  Instances For