The vector bundle of continuous (semi)linear maps #
We define the (topological) vector bundle of continuous (semi)linear maps between two vector bundles over the same base.
Given bundles E₁ E₂ : B → Type*
, normed spaces F₁
and F₂
, and a ring-homomorphism σ
between
their respective scalar fields, we define a vector bundle with fiber E₁ x →SL[σ] E₂ x
.
If the E₁
and E₂
are vector bundles with model fibers F₁
and F₂
, then this will be a
vector bundle with fiber F₁ →SL[σ] F₂
.
The topology on the total space is constructed from the trivializations for E₁
and E₂
and the
norm-topology on the model fiber F₁ →SL[𝕜] F₂
using the VectorPrebundle
construction. This is
a bit awkward because it introduces a dependence on the normed space structure of the model fibers,
rather than just their topological vector space structure; it is not clear whether this is
necessary.
Similar constructions should be possible (but are yet to be formalized) for tensor products of topological vector bundles, exterior algebras, and so on, where again the topology can be defined using a norm on the fiber model if this helps.
A reducible type synonym for the bundle of continuous (semi)linear maps.
Equations
- Bundle.ContinuousLinearMap σ E₁ E₂ x = (E₁ x →SL[σ] E₂ x)
Instances For
Assume eᵢ
and eᵢ'
are trivializations of the bundles Eᵢ
over base B
with fiber Fᵢ
(i ∈ {1,2}
), then Pretrivialization.continuousLinearMapCoordChange σ e₁ e₁' e₂ e₂'
is the
coordinate change function between the two induced (pre)trivializations
Pretrivialization.continuousLinearMap σ e₁ e₂
and
Pretrivialization.continuousLinearMap σ e₁' e₂'
of the bundle of continuous linear maps.
Equations
- Pretrivialization.continuousLinearMapCoordChange σ e₁ e₁' e₂ e₂' b = ↑((Trivialization.coordChangeL 𝕜₁ e₁' e₁ b).symm.arrowCongrSL (Trivialization.coordChangeL 𝕜₂ e₂ e₂' b))
Instances For
Given trivializations e₁
, e₂
for vector bundles E₁
, E₂
over a base B
,
Pretrivialization.continuousLinearMap σ e₁ e₂
is the induced pretrivialization for the
continuous σ
-semilinear maps from E₁
to E₂
. That is, the map which will later become a
trivialization, after the bundle of continuous semilinear maps is equipped with the right
topological vector bundle structure.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The continuous σ
-semilinear maps between two topological vector bundles form a
VectorPrebundle
(this is an auxiliary construction for the
VectorBundle
instance, in which the pretrivializations are collated but no topology
on the total space is yet provided).
Equations
- One or more equations did not get rendered due to their size.
Instances For
Topology on the total space of the continuous σ
-semilinear maps between two "normable" vector
bundles over the same base.
Equations
- Bundle.ContinuousLinearMap.topologicalSpaceTotalSpace σ F₁ E₁ F₂ E₂ = (Bundle.ContinuousLinearMap.vectorPrebundle σ F₁ E₁ F₂ E₂).totalSpaceTopology
The continuous σ
-semilinear maps between two vector bundles form a fiber bundle.
Equations
- Bundle.ContinuousLinearMap.fiberBundle σ F₁ E₁ F₂ E₂ = (Bundle.ContinuousLinearMap.vectorPrebundle σ F₁ E₁ F₂ E₂).toFiberBundle
The continuous σ
-semilinear maps between two vector bundles form a vector bundle.
Given trivializations e₁
, e₂
in the atlas for vector bundles E₁
, E₂
over a base B
,
the induced trivialization for the continuous σ
-semilinear maps from E₁
to E₂
,
whose base set is e₁.baseSet ∩ e₂.baseSet
.
Equations
Instances For
Consider a continuous map v : M → E₁
to a vector bundle, over a base map b₁ : M → B₁
, and
another basemap b₂ : M → B₂
. Given linear maps ϕ m : E₁ (b₁ m) → E₂ (b₂ m)
depending
continuously on m
, one can apply ϕ m
to g m
, and the resulting map is continuous.
Note that the continuity of ϕ
can not be always be stated as continuity of a map into a bundle,
as the pullback bundles b₁ *ᵖ E₁
and b₂ *ᵖ E₂
only have a nice topology when b₁
and b₂
are
globally continuous, but we want to apply this lemma with only local information. Therefore, we
formulate it using continuity of ϕ
read in coordinates.
Version for ContinuousWithinAt
. We also give a version for ContinuousAt
, but no version for
ContinuousOn
or Continuous
as our assumption, written in coordinates, only makes sense around
a point.
For a version with B₁ = B₂
and b₁ = b₂
, in which continuity can be expressed without
inCoordinates
, see ContinuousWithinAt.clm_bundle_apply
Consider a continuous map v : M → E₁
to a vector bundle, over a base map b₁ : M → B₁
, and
another basemap b₂ : M → B₂
. Given linear maps ϕ m : E₁ (b₁ m) → E₂ (b₂ m)
depending
continuously on m
, one can apply ϕ m
to g m
, and the resulting map is continuous.
Note that the continuity of ϕ
can not be always be stated as continuity of a map into a bundle,
as the pullback bundles b₁ *ᵖ E₁
and b₂ *ᵖ E₂
only have a nice topology when b₁
and b₂
are
globally continuous, but we want to apply this lemma with only local information. Therefore, we
formulate it using continuity of ϕ
read in coordinates.
Version for ContinuousAt
. We also give a version for ContinuousWithinAt
, but no version for
ContinuousOn
or Continuous
as our assumption, written in coordinates, only makes sense around
a point.
For a version with B₁ = B₂
and b₁ = b₂
, in which continuity can be expressed without
inCoordinates
, see ContinuousWithinAt.clm_bundle_apply
Consider a C^n
map v : M → E₁
to a vector bundle, over a basemap b : M → B
, and
linear maps ϕ m : E₁ (b m) → E₂ (b m)
depending smoothly on m
.
One can apply ϕ m
to v m
, and the resulting map is C^n
.
Consider a C^n
map v : M → E₁
to a vector bundle, over a basemap b : M → B
, and
linear maps ϕ m : E₁ (b m) → E₂ (b m)
depending smoothly on m
.
One can apply ϕ m
to v m
, and the resulting map is C^n
.
Consider a C^n
map v : M → E₁
to a vector bundle, over a basemap b : M → B
, and
linear maps ϕ m : E₁ (b m) → E₂ (b m)
depending smoothly on m
.
One can apply ϕ m
to v m
, and the resulting map is C^n
.
Consider a C^n
map v : M → E₁
to a vector bundle, over a basemap b : M → B
, and
linear maps ϕ m : E₁ (b m) → E₂ (b m)
depending smoothly on m
.
One can apply ϕ m
to v m
, and the resulting map is C^n
.
Consider C^n
maps v : M → E₁
and v : M → E₂
to vector bundles, over a basemap
b : M → B
, and bilinear maps ψ m : E₁ (b m) → E₂ (b m) → E₃ (b m)
depending smoothly on m
.
One can apply ψ m
to v m
and w m
, and the resulting map is C^n
.
Consider C^n
maps v : M → E₁
and v : M → E₂
to vector bundles, over a basemap
b : M → B
, and bilinear maps ψ m : E₁ (b m) → E₂ (b m) → E₃ (b m)
depending smoothly on m
.
One can apply ψ m
to v m
and w m
, and the resulting map is C^n
.
Consider C^n
maps v : M → E₁
and v : M → E₂
to vector bundles, over a basemap
b : M → B
, and bilinear maps ψ m : E₁ (b m) → E₂ (b m) → E₃ (b m)
depending smoothly on m
.
One can apply ψ m
to v m
and w m
, and the resulting map is C^n
.
Consider C^n
maps v : M → E₁
and v : M → E₂
to vector bundles, over a basemap
b : M → B
, and bilinear maps ψ m : E₁ (b m) → E₂ (b m) → E₃ (b m)
depending smoothly on m
.
One can apply ψ m
to v m
and w m
, and the resulting map is C^n
.
Rewrite ContinuousLinearMap.inCoordinates
using continuous linear equivalences, in the
bundle of bilinear maps.