Documentation

Mathlib.Geometry.Manifold.Sheaf.LocallyRingedSpace

Smooth manifolds as locally ringed spaces #

This file equips a smooth manifold with the structure of a locally ringed space.

Main results #

Main definitions #

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)) :
IsUnit f ↔ f βˆ‰ RingHom.ker (eval IM (modelWithCornersSelf π•œ π•œ) M π•œ 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
Instances For