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).
- carrier : TopCat
- presheaf : TopCat.Presheaf CommRingCat ↑s.toPresheafedSpace
- IsSheaf : TopCat.Presheaf.IsSheaf s.presheaf
- localRing : ∀ (x : ↑↑s.toPresheafedSpace), LocalRing ↑(TopCat.Presheaf.stalk s.presheaf x)
Stalks of a locally ringed space are local rings.
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
The structure sheaf of a locally ringed space.
Instances For
- val : X.toSheafedSpace ⟶ Y.toSheafedSpace
the underlying morphism between ringed spaces
- prop : ∀ (x : ↑↑X.toPresheafedSpace), IsLocalRingHom (AlgebraicGeometry.PresheafedSpace.stalkMap s.val x)
the underlying morphism induces a local ring homomorphism on stalks
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
The identity morphism on a locally ringed space.
Instances For
Composition of morphisms of locally ringed spaces.
Instances For
The category of locally ringed spaces.
The forgetful functor from LocallyRingedSpace
to SheafedSpace CommRing
.
Instances For
The forgetful functor from LocallyRingedSpace
to Top
.
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
The restriction of a locally ringed space along an open embedding.
Instances For
The canonical map from the restriction to the supspace.
Instances For
The restriction of a locally ringed space X
to the top subspace is isomorphic to X
itself.