Smooth manifolds as locally ringed spaces #
This file equips a smooth manifold with the structure of a locally ringed space.
Main results #
smoothSheafCommRing.isUnit_stalk_iff: The units of the stalk atxof the sheaf of smooth functions from a smooth manifoldMto its scalar fieldπ, considered as a sheaf of commutative rings, are the functions whose values atxare nonzero.
Main definitions #
IsManifold.locallyRingedSpace: A smooth manifold can be considered as a locally ringed space.
TODO #
Characterize morphisms-of-locally-ringed-spaces (AlgebraicGeometry.LocallyRingedSpace.Hom) between
smooth manifolds.
theorem
smoothSheafCommRing.isUnit_stalk_iff
{π : Type u}
[NontriviallyNormedField π]
{EM : Type u_1}
[NormedAddCommGroup EM]
[NormedSpace π EM]
{HM : Type u_2}
[TopologicalSpace HM]
(IM : ModelWithCorners π EM HM)
{M : Type u}
[TopologicalSpace M]
[ChartedSpace HM M]
{x : M}
(f : β((smoothSheafCommRing IM (modelWithCornersSelf π π) M π).presheaf.stalk x))
:
The units of the stalk at x of the sheaf of smooth functions from M to π, considered as a
sheaf of commutative rings, are the functions whose values at x are nonzero.
theorem
smoothSheafCommRing.nonunits_stalk
{π : Type u}
[NontriviallyNormedField π]
{EM : Type u_1}
[NormedAddCommGroup EM]
[NormedSpace π EM]
{HM : Type u_2}
[TopologicalSpace HM]
(IM : ModelWithCorners π EM HM)
{M : Type u}
[TopologicalSpace M]
[ChartedSpace HM M]
(x : M)
:
nonunits β((smoothSheafCommRing IM (modelWithCornersSelf π π) M π).presheaf.stalk x) = β(RingHom.ker (eval IM (modelWithCornersSelf π π) M π x))
The non-units of the stalk at x of the sheaf of smooth functions from M to π, considered
as a sheaf of commutative rings, are the functions whose values at x are zero.
instance
smoothSheafCommRing.instLocalRing_stalk
{π : Type u}
[NontriviallyNormedField π]
{EM : Type u_1}
[NormedAddCommGroup EM]
[NormedSpace π EM]
{HM : Type u_2}
[TopologicalSpace HM]
(IM : ModelWithCorners π EM HM)
{M : Type u}
[TopologicalSpace M]
[ChartedSpace HM M]
(x : M)
:
IsLocalRing β((smoothSheafCommRing IM (modelWithCornersSelf π π) M π).presheaf.stalk x)
The stalks of the structure sheaf of a smooth manifold are local rings.
def
IsManifold.locallyRingedSpace
{π : Type u}
[NontriviallyNormedField π]
{EM : Type u_1}
[NormedAddCommGroup EM]
[NormedSpace π EM]
{HM : Type u_2}
[TopologicalSpace HM]
(IM : ModelWithCorners π EM HM)
(M : Type u)
[TopologicalSpace M]
[ChartedSpace HM M]
:
A smooth manifold can be considered as a locally ringed space.
Equations
- IsManifold.locallyRingedSpace IM M = { carrier := { carrier := M, str := instβΒΉ }, presheaf := smoothPresheafCommRing IM (modelWithCornersSelf π π) M π, IsSheaf := β―, isLocalRing := β― }