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:
- the set of charts, which is data
- the fact that changes of charts belong to some group (in fact groupoid), which is additional Prop.
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
structure_groupoid H
: a subset of local homeomorphisms ofH
stable under composition, inverse and restriction (ex: local diffeos).continuous_groupoid H
: the groupoid of all local homeomorphisms ofH
charted_space H M
: charted space structure onM
modelled onH
, given by an atlas of local homeomorphisms fromM
toH
whose sources coverM
. This is a type class.has_groupoid M G
: whenG
is a structure groupoid onH
andM
is a charted space modelled onH
, require that all coordinate changes belong toG
. This is a type class.atlas H M
: whenM
is a charted space modelled onH
, the atlas of this charted space structure, i.e., the set of charts.G.maximal_atlas M
: whenM
is a charted space modelled onH
and admittingG
as a structure groupoid, one can consider all the local homeomorphisms fromM
toH
such that changing coordinate from any chart to them belongs toG
. This is a larger atlas, called the maximal atlas (for the groupoidG
).structomorph G M M'
: the type of diffeomorphisms between the charted spacesM
andM'
for the groupoidG
. We avoid the word diffeomorphism, keeping it for the smooth category.
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:
pregroupoid H
: a subset of local mas ofH
stable under composition and restriction, but not inverse (ex: smooth maps)groupoid_of_pregroupoid
: construct a groupoid from a pregroupoid, by requiring that a map and its inverse both belong to the pregroupoid (ex: construct diffeos from smooth maps)chart_at H x
is a preferred chart atx : M
whenM
has a charted space structure modelled onH
.G.compatible he he'
states that, for any two chartse
ande'
in the atlas, the composition ofe.symm
ande'
belongs to the groupoidG
whenM
admitsG
as a structure groupoid.G.compatible_of_mem_maximal_atlas he he'
states that, for any two chartse
ande'
in the maximal atlas associated to the groupoidG
, the composition ofe.symm
ande'
belongs to theG
ifM
admitsG
as a structure groupoid.charted_space_core.to_charted_space
: consider a space without a topology, but endowed with a set of charts (which are local equivs) for which the change of coordinates are local homeos. Then one can construct a topology on the space for which the charts become local homeos, defining a genuine charted space structure.
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
.
- members : set (local_homeomorph H H)
- trans' : ∀ (e e' : local_homeomorph H H), e ∈ c.members → e' ∈ c.members → e.trans e' ∈ c.members
- symm' : ∀ (e : local_homeomorph H H), e ∈ c.members → e.symm ∈ c.members
- id_mem' : local_homeomorph.refl H ∈ c.members
- locality' : ∀ (e : local_homeomorph H H), (∀ (x : H), x ∈ e.to_local_equiv.source → (∃ (s : set H), is_open s ∧ x ∈ s ∧ e.restr s ∈ c.members)) → e ∈ c.members
- eq_on_source' : ∀ (e e' : local_homeomorph H H), e ∈ c.members → e' ≈ e → e' ∈ c.members
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.
Equations
- structure_groupoid.has_mem = {mem := λ (e : local_homeomorph H H) (G : structure_groupoid H), e ∈ G.members}
Partial order on the set of groupoids, given by inclusion of the members of the groupoid
Equations
- structure_groupoid.partial_order = partial_order.lift structure_groupoid.members structure_groupoid.partial_order._proof_1
The trivial groupoid, containing only the identity (and maps with empty source, as this is necessary from the definition)
Equations
- id_groupoid H = {members := {local_homeomorph.refl H} ∪ {e : local_homeomorph H H | e.to_local_equiv.source = ∅}, trans' := _, symm' := _, id_mem' := _, locality' := _, eq_on_source' := _}
Every structure groupoid contains the identity groupoid
Equations
- structure_groupoid.order_bot = {bot := id_groupoid H _inst_1, le := partial_order.le structure_groupoid.partial_order, lt := partial_order.lt structure_groupoid.partial_order, le_refl := _, le_trans := _, lt_iff_le_not_le := _, le_antisymm := _, bot_le := _}
Equations
- structure_groupoid.inhabited H = {default := id_groupoid H _inst_2}
- property : (H → H) → set H → Prop
- comp : ∀ {f g : H → H} {u v : set H}, c.property f u → c.property g v → is_open u → is_open v → is_open (u ∩ f ⁻¹' v) → c.property (g ∘ f) (u ∩ f ⁻¹' v)
- id_mem : c.property id set.univ
- locality : ∀ {f : H → H} {u : set H}, is_open u → (∀ (x : H), x ∈ u → (∃ (v : set H), is_open v ∧ x ∈ v ∧ c.property f (u ∩ v))) → c.property f u
- congr : ∀ {f g : H → H} {u : set H}, is_open u → (∀ (x : H), x ∈ u → g x = f x) → c.property f u → c.property g u
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
- PG.groupoid = {members := {e : local_homeomorph H H | PG.property ⇑e e.to_local_equiv.source ∧ PG.property ⇑(e.symm) e.to_local_equiv.target}, trans' := _, symm' := _, id_mem' := _, locality' := _, eq_on_source' := _}
The pregroupoid of all local maps on a topological space H
Equations
- pregroupoid.inhabited H = {default := continuous_pregroupoid H _inst_2}
The groupoid of all local homeomorphisms on a topological space H
Equations
Every structure groupoid is contained in the groupoid of all local homeomorphisms
Equations
- structure_groupoid.order_top = {top := continuous_groupoid H _inst_1, le := partial_order.le structure_groupoid.partial_order, lt := partial_order.lt structure_groupoid.partial_order, le_refl := _, le_trans := _, lt_iff_le_not_le := _, le_antisymm := _, le_top := _}
The trivial restriction-closed groupoid, containing only local homeomorphisms equivalent to the restriction of the identity to the various open subsets.
Equations
- id_restr_groupoid = {members := {e : local_homeomorph H H | ∃ {s : set H} (h : is_open s), e ≈ local_homeomorph.of_set s h}, trans' := _, symm' := _, id_mem' := _, locality' := _, eq_on_source' := _}
The trivial restriction-closed groupoid is indeed closed_under_restriction
.
Equations
A groupoid is closed under restriction if and only if it contains the trivial restriction-closed groupoid.
The groupoid of all local homeomorphisms on a topological space H
is closed under restriction.
Equations
Charted spaces
- atlas : set (local_homeomorph M H)
- chart_at : M → local_homeomorph M H
- mem_chart_source : ∀ (x : M), x ∈ (charted_space.chart_at H x).to_local_equiv.source
- chart_mem_atlas : ∀ (x : M), charted_space.chart_at H x ∈ charted_space.atlas H M
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)
.
Any space is a charted_space modelled over itself, by just using the identity chart
Equations
- charted_space_self H = {atlas := {local_homeomorph.refl H}, chart_at := λ (x : H), local_homeomorph.refl H, mem_chart_source := _, chart_mem_atlas := _}
In the trivial charted_space structure of a space modelled over itself through the identity, the atlas members are just the identity
In the model space, chart_at is always the identity
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
- model_prod H H' = (H × H')
Equations
- model_prod_inhabited = {default := (inhabited.default α _inst_1, inhabited.default β _inst_2)}
Equations
The product of two charted spaces is naturally a charted space, with the canonical construction of the atlas of product maps.
Equations
- prod_charted_space H M H' M' = {atlas := {f : local_homeomorph (M × M') (model_prod H H') | ∃ (g : local_homeomorph M H) (H_1 : g ∈ charted_space.atlas H M) (h : local_homeomorph M' H') (H_1 : h ∈ charted_space.atlas H' M'), f = g.prod h}, chart_at := λ (x : M × M'), (charted_space.chart_at H x.fst).prod (charted_space.chart_at H' x.snd), mem_chart_source := _, chart_mem_atlas := _}
Constructing a topology from an atlas
- atlas : set (local_equiv M H)
- chart_at : M → local_equiv M H
- mem_chart_source : ∀ (x : M), x ∈ (c.chart_at x).source
- chart_mem_atlas : ∀ (x : M), c.chart_at x ∈ c.atlas
- open_source : ∀ (e e' : local_equiv M H), e ∈ c.atlas → e' ∈ c.atlas → is_open (e.symm.trans e').source
- continuous_to_fun : ∀ (e e' : local_equiv M H), e ∈ c.atlas → e' ∈ c.atlas → continuous_on ⇑(e.symm.trans e') (e.symm.trans e').source
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
- c.to_topological_space = topological_space.generate_from (⋃ (e : local_equiv M H) (he : e ∈ c.atlas) (s : set H) (s_open : is_open s), {⇑e ⁻¹' s ∩ e.source})
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
- c.local_homeomorph e he = {to_local_equiv := {to_fun := e.to_fun, inv_fun := e.inv_fun, source := e.source, target := e.target, map_source' := _, map_target' := _, left_inv' := _, right_inv' := _}, open_source := _, open_target := _, continuous_to_fun := _, continuous_inv_fun := _}
Given a charted space without topology, endow it with a genuine charted space structure with respect to the topology constructed from the atlas.
Equations
- c.to_charted_space = {atlas := ⋃ (e : local_equiv M H) (he : e ∈ c.atlas), {c.local_homeomorph e he}, chart_at := λ (x : M), c.local_homeomorph (c.chart_at x) _, mem_chart_source := _, chart_mem_atlas := _}
Charted space with a given structure groupoid
- compatible : ∀ {e e' : local_homeomorph M H}, e ∈ charted_space.atlas H M → e' ∈ charted_space.atlas H M → e.symm.trans e' ∈ G
A charted space has an atlas in a groupoid G
if the change of coordinates belong to the
groupoid
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.
The trivial charted space structure on the model space is compatible with any groupoid
Equations
- _ = _
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
- structure_groupoid.maximal_atlas M G = {e : local_homeomorph M H | ∀ (e' : local_homeomorph M H), e' ∈ charted_space.atlas H M → e.symm.trans e' ∈ G ∧ e'.symm.trans e ∈ G}
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.
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
- singleton_charted_space e h = {atlas := {e}, chart_at := λ (_x : α), e, mem_chart_source := _, chart_mem_atlas := _}
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.
An open subset of a charted space is naturally a charted space.
Equations
- s.charted_space = {atlas := ⋃ (x : ↥s), {(charted_space.chart_at H x.val).subtype_restr s}, chart_at := λ (x : ↥s), (charted_space.chart_at H x.val).subtype_restr s, mem_chart_source := _, chart_mem_atlas := _}
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
- to_homeomorph : M ≃ₜ M'
- mem_groupoid : ∀ (c_1 : local_homeomorph M H) (c' : local_homeomorph M' H), c_1 ∈ charted_space.atlas H M → c' ∈ charted_space.atlas H M' → c_1.symm.trans (c.to_homeomorph.to_local_homeomorph.trans c') ∈ G
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.
The identity is a diffeomorphism of any charted space, for any groupoid.
Equations
- structomorph.refl M = {to_homeomorph := {to_equiv := (homeomorph.refl M).to_equiv, continuous_to_fun := _, continuous_inv_fun := _}, mem_groupoid := _}
The inverse of a structomorphism is a structomorphism
Equations
- e.symm = {to_homeomorph := {to_equiv := e.to_homeomorph.symm.to_equiv, continuous_to_fun := _, continuous_inv_fun := _}, mem_groupoid := _}
The composition of structomorphisms is a structomorphism
Equations
- e.trans e' = {to_homeomorph := {to_equiv := (e.to_homeomorph.trans e'.to_homeomorph).to_equiv, continuous_to_fun := _, continuous_inv_fun := _}, mem_groupoid := _}