mathlib documentation

geometry.​manifold.​charted_space

geometry.​manifold.​charted_space

Charted spaces

A smooth manifold is a topological space M locally modelled on a euclidean space (or a euclidean half-space for manifolds with boundaries, or an infinite dimensional vector space for more general notions of manifolds), i.e., the manifold is covered by open subsets on which there are local homeomorphisms (the charts) going to a model space H, and the changes of charts should be smooth maps.

In this file, we introduce a general framework describing these notions, where the model space is an arbitrary topological space. We avoid the word manifold, which should be reserved for the situation where the model space is a (subset of a) vector space, and use the terminology charted space instead.

If the changes of charts satisfy some additional property (for instance if they are smooth), then M inherits additional structure (it makes sense to talk about smooth manifolds). There are therefore two different ingredients in a charted space:

We separate these two parts in the definition: the charted space structure is just the set of charts, and then the different smoothness requirements (smooth manifold, orientable manifold, contact manifold, and so on) are additional properties of these charts. These properties are formalized through the notion of structure groupoid, i.e., a set of local homeomorphisms stable under composition and inverse, to which the change of coordinates should belong.

Main definitions

As a basic example, we give the instance instance charted_space_model_space (H : Type*) [topological_space H] : charted_space H H saying that a topological space is a charted space over itself, with the identity as unique chart. This charted space structure is compatible with any groupoid.

Additional useful definitions:

Implementation notes

The atlas in a charted space is not a maximal atlas in general: the notion of maximality depends on the groupoid one considers, and changing groupoids changes the maximal atlas. With the current formalization, it makes sense first to choose the atlas, and then to ask whether this precise atlas defines a smooth manifold, an orientable manifold, and so on. A consequence is that structomorphisms between M and M' do not induce a bijection between the atlases of M and M': the definition is only that, read in charts, the structomorphism locally belongs to the groupoid under consideration. (This is equivalent to inducing a bijection between elements of the maximal atlas). A consequence is that the invariance under structomorphisms of properties defined in terms of the atlas is not obvious in general, and could require some work in theory (amounting to the fact that these properties only depend on the maximal atlas, for instance). In practice, this does not create any real difficulty.

We use the letter H for the model space thinking of the case of manifolds with boundary, where the model space is a half space.

Manifolds are sometimes defined as topological spaces with an atlas of local diffeomorphisms, and sometimes as spaces with an atlas from which a topology is deduced. We use the former approach: otherwise, there would be an instance from manifolds to topological spaces, which means that any instance search for topological spaces would try to find manifold structures involving a yet unknown model space, leading to problems. However, we also introduce the latter approach, through a structure charted_space_core making it possible to construct a topology out of a set of local equivs with compatibility conditions (but we do not register it as an instance).

In the definition of a charted space, the model space is written as an explicit parameter as there can be several model spaces for a given topological space. For instance, a complex manifold (modelled over ℂ^n) will also be seen sometimes as a real manifold modelled over ℝ^(2n).

Notations

In the locale manifold, we denote the composition of local homeomorphisms with ≫ₕ, and the composition of local equivs with .

Structure groupoids

One could add to the definition of a structure groupoid the fact that the restriction of an element of the groupoid to any open set still belongs to the groupoid. (This is in Kobayashi-Nomizu.) I am not sure I want this, for instance on H × E where E is a vector space, and the groupoid is made of functions respecting the fibers and linear in the fibers (so that a charted space over this groupoid is naturally a vector bundle) I prefer that the members of the groupoid are always defined on sets of the form s × E. There is a typeclass closed_under_restriction for groupoids which have the restriction property.

The only nontrivial requirement is locality: if a local homeomorphism belongs to the groupoid around each point in its domain of definition, then it belongs to the groupoid. Without this requirement, the composition of structomorphisms does not have to be a structomorphism. Note that this implies that a local homeomorphism with empty source belongs to any structure groupoid, as it trivially satisfies this condition.

There is also a technical point, related to the fact that a local homeomorphism is by definition a global map which is a homeomorphism when restricted to its source subset (and its values outside of the source are not relevant). Therefore, we also require that being a member of the groupoid only depends on the values on the source.

We use primes in the structure names as we will reformulate them below (without primes) using a has_mem instance, writing e ∈ G instead of e ∈ G.members.

structure structure_groupoid (H : Type u) [topological_space H] :
Type u

A structure groupoid is a set of local homeomorphisms of a topological space stable under composition and inverse. They appear in the definition of the smoothness class of a manifold.

theorem structure_groupoid.​trans {H : Type u} [topological_space H] (G : structure_groupoid H) {e e' : local_homeomorph H H} :
e Ge' Ge.trans e' G

theorem structure_groupoid.​symm {H : Type u} [topological_space H] (G : structure_groupoid H) {e : local_homeomorph H H} :
e Ge.symm G

theorem structure_groupoid.​locality {H : Type u} [topological_space H] (G : structure_groupoid H) {e : local_homeomorph H H} :
(∀ (x : H), x e.to_local_equiv.source(∃ (s : set H), is_open s x s e.restr s G))e G

theorem structure_groupoid.​eq_on_source {H : Type u} [topological_space H] (G : structure_groupoid H) {e e' : local_homeomorph H H} :
e Ge' ee' G

@[instance]

Partial order on the set of groupoids, given by inclusion of the members of the groupoid

Equations
theorem structure_groupoid.​le_iff {H : Type u} [topological_space H] {G₁ G₂ : structure_groupoid H} :
G₁ G₂ ∀ (e : local_homeomorph H H), e G₁e G₂

The trivial groupoid, containing only the identity (and maps with empty source, as this is necessary from the definition)

Equations
structure pregroupoid (H : Type u_5) [topological_space H] :
Type u_5

To construct a groupoid, one may consider classes of local homeos such that both the function and its inverse have some property. If this property is stable under composition, one gets a groupoid. pregroupoid bundles the properties needed for this construction, with the groupoid of smooth functions with smooth inverses as an application.

Construct a groupoid of local homeos for which the map and its inverse have some property, from a pregroupoid asserting that this property is stable under composition.

Equations
theorem groupoid_of_pregroupoid_le {H : Type u} [topological_space H] (PG₁ PG₂ : pregroupoid H) :
(∀ (f : H → H) (s : set H), PG₁.property f sPG₂.property f s)PG₁.groupoid PG₂.groupoid

The pregroupoid of all local maps on a topological space H

Equations

The groupoid of all local homeomorphisms on a topological space H

Equations
@[instance]

Every structure groupoid is contained in the groupoid of all local homeomorphisms

Equations
@[class]
structure closed_under_restriction {H : Type u} [topological_space H] :

A groupoid is closed under restriction if it contains all restrictions of its element local homeomorphisms to open subsets of the source.

Instances
theorem closed_under_restriction' {H : Type u} [topological_space H] {G : structure_groupoid H} [closed_under_restriction G] {e : local_homeomorph H H} (he : e G) {s : set H} :
is_open se.restr s G

The trivial restriction-closed groupoid, containing only local homeomorphisms equivalent to the restriction of the identity to the various open subsets.

Equations

A groupoid is closed under restriction if and only if it contains the trivial restriction-closed groupoid.

@[instance]

The groupoid of all local homeomorphisms on a topological space H is closed under restriction.

Equations

Charted spaces

@[class]
structure charted_space (H : Type u_5) [topological_space H] (M : Type u_6) [topological_space M] :
Type (max u_5 u_6)

A charted space is a topological space endowed with an atlas, i.e., a set of local homeomorphisms taking value in a model space H, called charts, such that the domains of the charts cover the whole space. We express the covering property by chosing for each x a member chart_at H x of the atlas containing x in its source: in the smooth case, this is convenient to construct the tangent bundle in an efficient way. The model space is written as an explicit parameter as there can be several model spaces for a given topological space. For instance, a complex manifold (modelled over ℂ^n) will also be seen sometimes as a real manifold over ℝ^(2n).

Instances
@[instance]
def charted_space_self (H : Type u_1) [topological_space H] :

Any space is a charted_space modelled over itself, by just using the identity chart

Equations
@[simp]

In the trivial charted_space structure of a space modelled over itself through the identity, the atlas members are just the identity

@[simp]

In the model space, chart_at is always the identity

def model_prod  :
Type u_1Type u_2Type (max u_1 u_2)

Same thing as H × H'. We introduce it for technical reasons: a charted space M with model H is a set of local charts from M to H covering the space. Every space is registered as a charted space over itself, using the only chart id, in manifold_model_space. You can also define a product of charted space M and M' (with model space H × H') by taking the products of the charts. Now, on H × H', there are two charted space structures with model space H × H' itself, the one coming from manifold_model_space, and the one coming from the product of the two manifold_model_space on each component. They are equal, but not defeq (because the product of id and id is not defeq to id), which is bad as we know. This expedient of renaming H × H' solves this problem.

Equations
@[instance]
def model_prod_inhabited {α : Type u_1} {β : Type u_2} [inhabited α] [inhabited β] :

Equations
@[simp]
theorem model_prod_range_prod_id {H : Type u_1} {H' : Type u_2} {α : Type u_3} (f : H → α) :
set.range (λ (p : model_prod H H'), (f p.fst, p.snd)) = (set.range f).prod set.univ

@[instance]
def prod_charted_space (H : Type u_1) [topological_space H] (M : Type u_2) [topological_space M] [charted_space H M] (H' : Type u_3) [topological_space H'] (M' : Type u_4) [topological_space M'] [charted_space H' M'] :

The product of two charted spaces is naturally a charted space, with the canonical construction of the atlas of product maps.

Equations
@[simp]
theorem prod_charted_space_chart_at {H : Type u} {H' : Type u_1} {M : Type u_2} {M' : Type u_3} [topological_space H] [topological_space M] [charted_space H M] [topological_space H'] [topological_space M'] [charted_space H' M'] {x : M × M'} :

Constructing a topology from an atlas

@[nolint]
structure charted_space_core (H : Type u_5) [topological_space H] :
Type u_6Type (max u_5 u_6)

Sometimes, one may want to construct a charted space structure on a space which does not yet have a topological structure, where the topology would come from the charts. For this, one needs charts that are only local equivs, and continuity properties for their composition. This is formalised in charted_space_core.

Topology generated by a set of charts on a Type.

Equations
theorem charted_space_core.​open_source' {H : Type u} {M : Type u_2} [topological_space H] (c : charted_space_core H M) {e : local_equiv M H} :

theorem charted_space_core.​open_target {H : Type u} {M : Type u_2} [topological_space H] (c : charted_space_core H M) {e : local_equiv M H} :

def charted_space_core.​local_homeomorph {H : Type u} {M : Type u_2} [topological_space H] (c : charted_space_core H M) (e : local_equiv M H) :

An element of the atlas in a charted space without topology becomes a local homeomorphism for the topology constructed from this atlas. The local_homeomorph version is given in this definition.

Equations
def charted_space_core.​to_charted_space {H : Type u} {M : Type u_2} [topological_space H] (c : charted_space_core H M) :

Given a charted space without topology, endow it with a genuine charted space structure with respect to the topology constructed from the atlas.

Equations

Charted space with a given structure groupoid

@[class]
structure has_groupoid {H : Type u_5} [topological_space H] (M : Type u_6) [topological_space M] [charted_space H M] :

A charted space has an atlas in a groupoid G if the change of coordinates belong to the groupoid

Instances
theorem structure_groupoid.​compatible {H : Type u_1} [topological_space H] (G : structure_groupoid H) {M : Type u_2} [topological_space M] [charted_space H M] [has_groupoid M G] {e e' : local_homeomorph M H} :

Reformulate in the structure_groupoid namespace the compatibility condition of charts in a charted space admitting a structure groupoid, to make it more easily accessible with dot notation.

theorem has_groupoid_of_le {H : Type u} {M : Type u_2} [topological_space H] [topological_space M] [charted_space H M] {G₁ G₂ : structure_groupoid H} :
has_groupoid M G₁G₁ G₂has_groupoid M G₂

theorem has_groupoid_of_pregroupoid {H : Type u} {M : Type u_2} [topological_space H] [topological_space M] [charted_space H M] (PG : pregroupoid H) :

@[instance]

The trivial charted space structure on the model space is compatible with any groupoid

Equations
  • _ = _
@[instance]

Any charted space structure is compatible with the groupoid of all local homeomorphisms

Equations

Given a charted space admitting a structure groupoid, the maximal atlas associated to this structure groupoid is the set of all local charts that are compatible with the atlas, i.e., such that changing coordinates with an atlas member gives an element of the groupoid.

Equations

The elements of the atlas belong to the maximal atlas for any structure groupoid

Changing coordinates between two elements of the maximal atlas gives rise to an element of the structure groupoid.

In the model space, the identity is in any maximal atlas.

def singleton_charted_space {H : Type u} [topological_space H] {α : Type u_5} [topological_space α] (e : local_homeomorph α H) :

If a single local homeomorphism e from a space α into H has source covering the whole space α, then that local homeomorphism induces an H-charted space structure on α. (This condition is equivalent to e being an open embedding of α into H; see local_homeomorph.to_open_embedding and open_embedding.to_local_homeomorph.)

Equations
theorem singleton_charted_space_one_chart {H : Type u} [topological_space H] {α : Type u_5} [topological_space α] (e : local_homeomorph α H) (h : e.to_local_equiv.source = set.univ) (e' : local_homeomorph α H) :
e' charted_space.atlas H αe' = e

Given a local homeomorphism e from a space α into H, if its source covers the whole space α, then the induced charted space structure on α is has_groupoid G for any structure groupoid G which is closed under restrictions.

@[instance]

An open subset of a charted space is naturally a charted space.

Equations
@[instance]

If a groupoid G is closed_under_restriction, then an open subset of a space which is has_groupoid G is naturally has_groupoid G.

Equations
  • _ = _

Structomorphisms

@[nolint]
structure structomorph {H : Type u} [topological_space H] (G : structure_groupoid H) (M : Type u_5) (M' : Type u_6) [topological_space M] [topological_space M'] [charted_space H M] [charted_space H M'] :
Type (max u_5 u_6)

A G-diffeomorphism between two charted spaces is a homeomorphism which, when read in the charts, belongs to G. We avoid the word diffeomorph as it is too related to the smooth category, and use structomorph instead.

def structomorph.​refl {H : Type u} [topological_space H] {G : structure_groupoid H} (M : Type u_1) [topological_space M] [charted_space H M] [has_groupoid M G] :

The identity is a diffeomorphism of any charted space, for any groupoid.

Equations
def structomorph.​symm {H : Type u} {M : Type u_2} {M' : Type u_3} [topological_space H] [topological_space M] [charted_space H M] [topological_space M'] {G : structure_groupoid H} [charted_space H M'] :
structomorph G M M'structomorph G M' M

The inverse of a structomorphism is a structomorphism

Equations
def structomorph.​trans {H : Type u} {M : Type u_2} {M' : Type u_3} {M'' : Type u_4} [topological_space H] [topological_space M] [charted_space H M] [topological_space M'] [topological_space M''] {G : structure_groupoid H} [charted_space H M'] [charted_space H M''] :
structomorph G M M'structomorph G M' M''structomorph G M M''

The composition of structomorphisms is a structomorphism

Equations