The groupoid of smooth, fiberwise-linear maps #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file contains preliminaries for the definition of a smooth vector bundle: an associated
structure_groupoid
, the groupoid of smooth_fiberwise_linear
functions.
The groupoid of smooth, fiberwise-linear maps #
For B
a topological space and F
a 𝕜
-normed space, a map from U : set B
to F ≃L[𝕜] F
determines a local homeomorphism from B × F
to itself by its action fiberwise.
Equations
- fiberwise_linear.local_homeomorph φ hU hφ h2φ = {to_local_equiv := {to_fun := λ (x : B × F), (x.fst, ⇑(φ x.fst) x.snd), inv_fun := λ (x : B × F), (x.fst, ⇑((φ x.fst).symm) x.snd), source := U ×ˢ set.univ, target := U ×ˢ set.univ, map_source' := _, map_target' := _, left_inv' := _, right_inv' := _}, open_source := _, open_target := _, continuous_to_fun := _, continuous_inv_fun := _}
Compute the composition of two local homeomorphisms induced by fiberwise linear equivalences.
Compute the source of the composition of two local homeomorphisms induced by fiberwise linear equivalences.
Compute the target of the composition of two local homeomorphisms induced by fiberwise linear equivalences.
Let e
be a local homeomorphism of B × F
. Suppose that at every point p
in the source of
e
, there is some neighbourhood s
of p
on which e
is equal to a bi-smooth fiberwise linear
local homeomorphism.
Then the source of e
is of the form U ×ˢ univ
, for some set U
in B
, and, at any point x
in
U
, admits a neighbourhood u
of x
such that e
is equal on u ×ˢ univ
to some bi-smooth
fiberwise linear local homeomorphism.
Let e
be a local homeomorphism of B × F
whose source is U ×ˢ univ
, for some set U
in
B
, and which, at any point x
in U
, admits a neighbourhood u
of x
such that e
is equal on
u ×ˢ univ
to some bi-smooth fiberwise linear local homeomorphism. Then e
itself is equal to
some bi-smooth fiberwise linear local homeomorphism.
This is the key mathematical point of the locality
condition in the construction of the
structure_groupoid
of bi-smooth fiberwise linear local homeomorphisms. The proof is by gluing
together the various bi-smooth fiberwise linear local homeomorphism which exist locally.
The U
in the conclusion is the same U
as in the hypothesis. We state it like this, because this
is exactly what we need for smooth_fiberwise_linear
.
For B
a manifold and F
a normed space, the groupoid on B × F
consisting of local
homeomorphisms which are bi-smooth and fiberwise linear, and induce the identity on B
.
When a (topological) vector bundle is smooth, then the composition of charts associated
to the vector bundle belong to this groupoid.
Equations
- smooth_fiberwise_linear B F IB = {members := ⋃ (φ : B → (F ≃L[𝕜] F)) (U : set B) (hU : is_open U) (hφ : smooth_on IB (model_with_corners_self 𝕜 (F →L[𝕜] F)) (λ (x : B), ↑(φ x)) U) (h2φ : smooth_on IB (model_with_corners_self 𝕜 (F →L[𝕜] F)) (λ (x : B), ↑((φ x).symm)) U), {e : local_homeomorph (B × F) (B × F) | e.eq_on_source (fiberwise_linear.local_homeomorph φ hU _ _)}, trans' := _, symm' := _, id_mem' := _, locality' := _, eq_on_source' := _}