Trivializations #
Main definitions #
Basic definitions #
-
Trivialization F p
: structure extending local homeomorphisms, defining a local trivialization of a topological spaceZ
with projectionp
and fiberF
. -
Pretrivialization F proj
: trivialization as a local equivalence, mainly used when the topology on the total space has not yet been defined.
Operations on bundles #
We provide the following operations on Trivialization
s.
Trivialization.compHomeomorph
: given a local trivializatione
of a fiber bundlep : Z → B
and a homeomorphismh : Z' ≃ₜ Z
, returns a local trivialization of the fiber bundlep ∘ h
.
Implementation notes #
Previously, in mathlib, there was a structure topological_vector_bundle.trivialization
which
extended another structure topological_fiber_bundle.trivialization
by a linearity hypothesis. As
of PR leanprover-community/mathlib#17359, we have changed this to a single structure
Trivialization
(no namespace), together with a mixin class Trivialization.IsLinear
.
This permits all the data of a vector bundle to be held at the level of fiber bundles, so that the
same trivializations can underlie an object's structure as (say) a vector bundle over ℂ
and as a
vector bundle over ℝ
, as well as its structure simply as a fiber bundle.
This might be a little surprising, given the general trend of the library to ever-increased bundling. But in this case the typical motivation for more bundling does not apply: there is no algebraic or order structure on the whole type of linear (say) trivializations of a bundle. Indeed, since trivializations only have meaning on their base sets (taking junk values outside), the type of linear trivializations is not even particularly well-behaved.
- toFun : Z → B × F
- invFun : B × F → Z
- source : Set Z
- map_target' : ∀ ⦃x : B × F⦄, x ∈ s.target → LocalEquiv.invFun s.toLocalEquiv x ∈ s.source
- left_inv' : ∀ ⦃x : Z⦄, x ∈ s.source → LocalEquiv.invFun s.toLocalEquiv (↑s.toLocalEquiv x) = x
- right_inv' : ∀ ⦃x : B × F⦄, x ∈ s.target → ↑s.toLocalEquiv (LocalEquiv.invFun s.toLocalEquiv x) = x
- open_target : IsOpen s.target
- baseSet : Set B
- open_baseSet : IsOpen s.baseSet
This structure contains the information left for a local trivialization (which is implemented
below as Trivialization F proj
) if the total space has not been given a topology, but we
have a topology on both the fiber and the base space. Through the construction
topological_fiber_prebundle F proj
it will be possible to promote a
Pretrivialization F proj
to a Trivialization F proj
.
Instances For
Coercion of a pretrivialization to a function. We don't use e.toFun
in the CoeFun
instance
because it is actually e.toLocalEquiv.toFun
, so simp
will apply lemmas about
toLocalEquiv
. While we may want to switch to this behavior later, doing it mid-port will break a
lot of proofs.
Instances For
If the fiber is nonempty, then the projection to
Composition of inverse and coercion from the subtype of the target.
Instances For
A fiberwise inverse to e
. This is the function F → E b
that induces a local inverse
B × F → TotalSpace F E
of e
on e.baseSet
. It is defined to be 0
outside e.baseSet
.
Instances For
- toFun : Z → B × F
- invFun : B × F → Z
- source : Set Z
- map_target' : ∀ ⦃x : B × F⦄, x ∈ s.target → LocalEquiv.invFun s.toLocalEquiv x ∈ s.source
- left_inv' : ∀ ⦃x : Z⦄, x ∈ s.source → LocalEquiv.invFun s.toLocalEquiv (↑s.toLocalEquiv x) = x
- right_inv' : ∀ ⦃x : B × F⦄, x ∈ s.target → ↑s.toLocalEquiv (LocalEquiv.invFun s.toLocalEquiv x) = x
- open_source : IsOpen s.source
- open_target : IsOpen s.target
- continuous_toFun : ContinuousOn (↑s.toLocalEquiv) s.source
- continuous_invFun : ContinuousOn s.invFun s.target
- baseSet : Set B
- open_baseSet : IsOpen s.baseSet
A structure extending local homeomorphisms, defining a local trivialization of a projection
proj : Z → B
with fiber F
, as a local homeomorphism between Z
and B × F
defined between two
sets of the form proj ⁻¹' baseSet
and baseSet × F
, acting trivially on the first coordinate.
Instances For
Coercion of a trivialization to a function. We don't use e.toFun
in the CoeFun
instance
because it is actually e.toLocalEquiv.toFun
, so simp
will apply lemmas about
toLocalEquiv
. While we may want to switch to this behavior later, doing it mid-port will break a
lot of proofs.
Instances For
Natural identification as a Pretrivialization
.
Instances For
The preimage of a subset of the base set is homeomorphic to the product with the fiber.
Instances For
The source is homeomorphic to the product of the base set with the fiber.
Instances For
Each fiber of a trivialization is homeomorphic to the specified fiber.
Instances For
In the domain of a bundle trivialization, the projection is continuous
Composition of a Trivialization
and a Homeomorph
.
Instances For
Read off the continuity of a function f : Z → X
at z : Z
by transferring via a
trivialization of Z
containing z
.
Read off the continuity of a function f : X → Z
at x : X
by transferring via a
trivialization of Z
containing f x
.
A fiberwise inverse to e'
. The function F → E x
that induces a local inverse
B × F → TotalSpace F E
of e'
on e'.baseSet
. It is defined to be 0
outside e'.baseSet
.
Instances For
If e
is a Trivialization
of proj : Z → B
with fiber F
and h
is a homeomorphism
F ≃ₜ F'
, then e.trans_fiber_homeomorph h
is the trivialization of proj
with the fiber F'
that sends p : Z
to ((e p).1, h (e p).2)
.
Instances For
Coordinate transformation in the fiber induced by a pair of bundle trivializations. See also
Trivialization.coordChangeHomeomorph
for a version bundled as F ≃ₜ F
.
Instances For
Coordinate transformation in the fiber induced by a pair of bundle trivializations, as a homeomorphism.
Instances For
Restrict a Trivialization
to an open set in the base.
Instances For
Given two bundle trivializations e
, e'
of proj : Z → B
and a set s : Set B
such that
the base sets of e
and e'
intersect frontier s
on the same set and e p = e' p
whenever
proj p ∈ e.baseSet ∩ frontier s
, e.piecewise e' s Hs Heq
is the bundle trivialization over
Set.ite s e.baseSet e'.baseSet
that is equal to e
on proj ⁻¹ s
and is equal to e'
otherwise.
Instances For
Given two bundle trivializations e
, e'
of a topological fiber bundle proj : Z → B
over a linearly ordered base B
and a point a ∈ e.baseSet ∩ e'.baseSet
such that
e
equals e'
on proj ⁻¹' {a}
, e.piecewise_le_of_eq e' a He He' Heq
is the bundle
trivialization over Set.ite (Iic a) e.baseSet e'.baseSet
that is equal to e
on points p
such that proj p ≤ a
and is equal to e'
otherwise.
Instances For
Given two bundle trivializations e
, e'
of a topological fiber bundle proj : Z → B
over a
linearly ordered base B
and a point a ∈ e.baseSet ∩ e'.baseSet
, e.piecewise_le e' a He He'
is the bundle trivialization over Set.ite (Iic a) e.baseSet e'.baseSet
that is equal to e
on
points p
such that proj p ≤ a
and is equal to ((e' p).1, h (e' p).2)
otherwise, where
h = e'.coord_change_homeomorph e _ _
is the homeomorphism of the fiber such that
h (e' p).2 = (e p).2
whenever e p = a
.
Instances For
Given two bundle trivializations e
, e'
over disjoint sets, e.disjoint_union e' H
is the
bundle trivialization over the union of the base sets that agrees with e
and e'
over their
base sets.