Local frames in a vector bundle #
Let V → M be a finite rank smooth vector bundle with standard fiber F.
A family of sections s i of V → M is called a C^k local frame on a set U ⊆ M iff each
section s i is C^k on U, and the section values s i x form a basis for each x ∈ U.
We define a predicate IsLocalFrame for a collection of sections to be a local frame on a set,
and define basic notions (such as the coefficients of a section w.r.t. a local frame, and
checking the smoothness of t via its coefficients in a local frame).
In future work, given a basis b for F and a local trivialisation e for V,
we will construct a smooth local frame on V w.r.t. e and b,
i.e. a collection of sections sᵢ of V which is smooth on e.baseSet such that {sᵢ x} is a
basis of V x for each x ∈ e.baseSet. Any section s of e can be uniquely written as
s = ∑ i, f^i sᵢ near x, and s is smooth at x iff the functions f^i are.
In this file, we prove the latter statement for finite-rank bundles (with coefficients in a
complete field). In OrthonormalFrame.lean, we will prove the same for real vector bundles of any
rank which admit a C^n bundle metric. This includes bundles of finite rank, modelled on a Hilbert
space or on a Banach space which has smooth partitions of unity.
We will use this to construct local extensions of a vector to a section which is smooth on the trivialisation domain.
Main definitions and results #
IsLocalFrameOn: a family of sectionss iofV → Mis called a C^k local frame on a setU ⊆ Miff each sections iisC^konU, and the section valuess i xform a basis for eachx ∈ U
Suppose {sᵢ} is a local frame on U, and hs : IsLocalFrameOn s U.
IsLocalFrameOn.toBasisAt hs: for eachx ∈ U, the vectorssᵢ xform a basis ofFIsLocalFrameOn.coeff hsdescribes the coefficient of sections ofVw.r.t.{sᵢ}.hs.coeff iis a linear map from sections ofVto functionsM → 𝕜.IsLocalFrameOn.eventually_eq_sum_coeff_smul hs: for a local frame{sᵢ}nearx, for each sectiontwe havet = ∑ i, (hs.coeff i t) • sᵢ.IsLocalFrameOn.coeff_sum_eq hs t hxproves thatt x = ∑ i, (hs.coeff i t) x • sᵢ x, provided thathx : x ∈ U.IsLocalFrameOn.coeff_congr hs: the coefficienths.coeff ioftin the local frame{sᵢ}only depends ontatx.IsLocalFrameOn.eq_iff_coeff hs: two sectionstandt'are equal atxif and only if their coefficients atxw.r.t.{sᵢ}agree.IsLocalFrameOn.contMDiffOn_of_coeff hs: a sectiontisC^konUif each coefficienths.coeff i tisC^konUIsLocalFrameOn.contMDiffAt_of_coeff hs: a sectiontisC^katx ∈ Uif all of its frame coefficients areIsLocalFrameOn.contMDiffOn_off_coeff hs: a sectiontisC^kon an open sett ⊆ Uff all of its frame coefficients areMDifferentiableversions of the above three statements
TODO #
IsLocalFrameOn.contMDiffOn_coeff hs: iftis aC^ksection, each coefficienths.coeff i tisC^konUIsLocalFrameOn.contMDiffAt_iff_coeff hs: a sectiontisC^katx ∈ Uiff all of its frame coefficients areIsLocalFrameOn.contMDiffOn_iff_coeff hs: a sectiontisC^kon an open sett ⊆ Uiff all of its frame coefficients are- a
MDifferentiableversion of each of these
Implementation notes #
Local frames use the junk value pattern: they are defined on all of M, but their value is
only meaningful on the set on which they are a local frame.
Tags #
vector bundle, local frame, smoothness
A family of sections s i of V → M is called a C^k local frame on a set U ⊆ M iff
- the section values
s i xform a basis for eachx ∈ U, - each section
s iisC^konU.
- contMDiffOn (i : ι) : ContMDiffOn I (I.prod (modelWithCornersSelf 𝕜 F)) n (fun (x : M) => Bundle.TotalSpace.mk' F x (s i x)) u
Instances For
If s = s' on u and s i is a local frame on u, then so is s'.
Given a local frame {s i} on U ∋ x, returns the basis {s i} of V x
Equations
- hs.toBasisAt hx = Module.Basis.mk ⋯ ⋯
Instances For
Coefficients of a section s of V w.r.t. a local frame {s i} on u.
Outside of u, this returns the junk value 0.
Equations
Instances For
A local frame locally spans the space of sections for V: for each local frame s i on an open
set u around x, we have t = ∑ i, (hs.coeff i t) • (s i x) near x.
The coefficients of t in a local frame at x only depend on t at x.
If s and s' are local frames which are equal at x,
a section t has equal frame coefficients in them.
Two sections s and t are equal at x if and only if their coefficients w.r.t. some local
frame at x agree.
Given a local frame s i on u, if a section t has C^k coefficients on u w.r.t. s i,
then t is C^n on u.
Given a local frame s i on a neighbourhood u of x,
if a section t has C^k coefficients at x w.r.t. s i, then t is C^n at x.
Given a local frame s i on an open set u containing x, if a section t has C^k
coefficients at x ∈ u w.r.t. s i, then t is C^n at x.
Given a local frame s i on u, if a section t has differentiable coefficients on u
w.r.t. s i, then t is differentiable on u.
Given a local frame s i on a neighbourhood u of x, if a section t has differentiable
coefficients at x w.r.t. s i, then t is differentiable at x.
Given a local frame s i on open set u containing x, if a section t
has differentiable coefficients at x ∈ u w.r.t. s i, then t is differentiable at x.