Structure groupoids #
This file contains the definitions and properties of structure groupoids, i.e., sets of open partial
homeomorphisms stable under composition and inverse. These are used to define charted spaces (and
hence manifolds). See the file Mathlib.Geometry.Manifold.ChartedSpace for more details.
Main definitions #
StructureGroupoid H: a subset of open partial homeomorphisms ofHstable under composition, inverse and restriction (ex: partial diffeomorphisms).continuousGroupoid H: the groupoid of all open partial homeomorphisms ofH.
Additional useful definitions:
Pregroupoid H: a subset of partial maps ofHstable under composition and restriction, but not inverse (ex: smooth maps)Pregroupoid.groupoid: 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)
Notation #
In the scope Manifold, we denote the composition of open partial homeomorphisms with ≫ₕ, and the
composition of partial equivs with ≫.
Composing two open partial homeomorphisms, by restricting to the maximal domain where their
composition is well defined.
Within the Manifold namespace, there is the notation e ≫ₕ f for this.
Equations
- Manifold.«term_≫ₕ_» = Lean.ParserDescr.trailingNode `Manifold.«term_≫ₕ_» 100 101 (Lean.ParserDescr.binary `andthen (Lean.ParserDescr.symbol " ≫ₕ ") (Lean.ParserDescr.cat `term 100))
Instances For
Composing two partial equivs, by restricting to the maximal domain where their composition
is well defined.
Within the Manifold namespace, there is the notation e ≫ f for this.
Equations
- Manifold.«term_≫_» = Lean.ParserDescr.trailingNode `Manifold.«term_≫_» 100 101 (Lean.ParserDescr.binary `andthen (Lean.ParserDescr.symbol " ≫ ") (Lean.ParserDescr.cat `term 100))
Instances For
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 ClosedUnderRestriction for groupoids
which have the restriction property.
The only nontrivial requirement is locality: if an open partial 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 an open partial 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 an open partial 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
Membership instance, writing e ∈ G instead of e ∈ G.members.
A structure groupoid is a set of open partial homeomorphisms of a topological space stable under composition and inverse. They appear in the definition of the smoothness class of a manifold.
- members : Set (OpenPartialHomeomorph H H)
Members of the structure groupoid are open partial homeomorphisms.
- trans' (e e' : OpenPartialHomeomorph H H) : e ∈ self.members → e' ∈ self.members → e.trans e' ∈ self.members
Structure groupoids are stable under composition.
Structure groupoids are stable under inverse.
The identity morphism lies in the structure groupoid.
- locality' (e : OpenPartialHomeomorph H H) : (∀ x ∈ e.source, ∃ (s : Set H), IsOpen s ∧ x ∈ s ∧ e.restr s ∈ self.members) → e ∈ self.members
Let
ebe an open partial homeomorphism. If for everyx ∈ e.source, the restriction of e to some open set aroundxlies in the groupoid, thenelies in the groupoid. - mem_of_eqOnSource' (e e' : OpenPartialHomeomorph H H) : e ∈ self.members → e' ≈ e → e' ∈ self.members
Membership in a structure groupoid respects the equivalence of open partial homeomorphisms.
Instances For
Equations
- instMembershipOpenPartialHomeomorphStructureGroupoid = { mem := fun (G : StructureGroupoid H) (e : OpenPartialHomeomorph H H) => e ∈ G.members }
Equations
- instSetLikeStructureGroupoidOpenPartialHomeomorph H = { coe := fun (s : StructureGroupoid H) => s.members, coe_injective' := ⋯ }
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Partial order on the set of groupoids, given by inclusion of the members of the groupoid.
The trivial groupoid, containing only the identity (and maps with empty source, as this is necessary from the definition).
Equations
Instances For
Every structure groupoid contains the identity groupoid.
Equations
- instStructureGroupoidOrderBot = { bot := idGroupoid H, bot_le := ⋯ }
Equations
- instInhabitedStructureGroupoid = { default := idGroupoid H }
To construct a groupoid, one may consider classes of open partial homeomorphisms 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.
Property describing membership in this groupoid: the pregroupoid "contains" all functions
H → Hhaving the pregroupoid property on somes : Set H- comp {f g : H → H} {u v : Set H} : self.property f u → self.property g v → IsOpen u → IsOpen v → IsOpen (u ∩ f ⁻¹' v) → self.property (g ∘ f) (u ∩ f ⁻¹' v)
The pregroupoid property is stable under composition
Pregroupoids contain the identity map (on
univ)- locality {f : H → H} {u : Set H} : IsOpen u → (∀ x ∈ u, ∃ (v : Set H), IsOpen v ∧ x ∈ v ∧ self.property f (u ∩ v)) → self.property f u
The pregroupoid property is "local", in the sense that
fhas the pregroupoid property onuiff its restriction to each open subset ofuhas it
Instances For
Construct a groupoid of partial homeos for which the map and its inverse have some property, from a pregroupoid asserting that this property is stable under composition.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The pregroupoid of all partial maps on a topological space H.
Equations
Instances For
Equations
- instInhabitedPregroupoid H = { default := continuousPregroupoid H }
The groupoid of all open partial homeomorphisms on a topological space H.
Equations
Instances For
Every structure groupoid is contained in the groupoid of all open partial homeomorphisms.
Equations
- instStructureGroupoidOrderTop = { top := continuousGroupoid H, le_top := ⋯ }
Equations
- One or more equations did not get rendered due to their size.
A groupoid is closed under restriction if it contains all restrictions of its element local homeomorphisms to open subsets of the source.
Instances
The trivial restriction-closed groupoid, containing only open partial homeomorphisms equivalent to the restriction of the identity to the various open subsets.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The trivial restriction-closed groupoid is indeed ClosedUnderRestriction.
A groupoid is closed under restriction if and only if it contains the trivial restriction-closed groupoid.
The groupoid of all open partial homeomorphisms on a topological space H
is closed under restriction.