1-jet bundles #
This file contains the definition of the 1-jet bundle J¹(M, M'), also known as
OneJetBundle I M I' M'.
We also define
OneJetExt I I' f : M → J¹(M, M'): the 1-jet extensionj¹fof a mapf : M → M'
We prove
- If
fis smooth,j¹fis smooth. - If
x ↦ (f₁ x, f₂ x, ϕ₁ x) : N → J¹(M₁, M₂)andx ↦ (f₂ x, f₃ x, ϕ₂ x) : N → J¹(M₂, M₃)are smooth, then so isx ↦ (f₁ x, f₃ x, ϕ₂ x ∘ ϕ₁ x) : N → J¹(M₁, M₃).
Equations
- deleteme1 I I' = inferInstance
Equations
- deleteme2 I I' = inferInstance
The fibers of the one jet-bundle.
Equations
- OneJetSpace I I' p = ((⇑ContMDiffMap.fst *ᵖ (TangentSpace I)) p →L[𝕜] (⇑ContMDiffMap.snd *ᵖ (TangentSpace I')) p)
Instances For
Equations
Equations
Equations
- instFunLikeOneJetSpaceTangentSpaceFstSnd I I' p = { coe := fun (φ : OneJetSpace I I' p) => (↑φ).toFun, coe_injective' := ⋯ }
The space of one jets of maps between two smooth manifolds.
Defined in terms of Bundle.TotalSpace to be able to put a suitable topology on it.
Equations
- OneJetBundle I M I' M' = Bundle.TotalSpace (E →L[𝕜] E') (OneJetSpace I I')
Instances For
Equations
- instModuleOneJetSpace I I' M' x = id inferInstance
Equations
- instTopologicalSpaceOneJetBundle I M I' M' = id inferInstance
Equations
Equations
The tangent bundle projection on the basis is a continuous map.
Computing the value of a chart around v at point v' in J¹(M, M').
The last component equals the continuous linear map v'.2, composed on both sides by an
appropriate coordinate change function.
In J¹(M, M'), the source of a chart has a nice formula
In J¹(M, M'), the target of a chart has a nice formula
The constructor of OneJetBundle, in case Sigma.mk will not give the right type.
Instances For
The one-jet extension of a function
Equations
- oneJetExt I I' f x = OneJetBundle.mk x (f x) (mfderiv I I' f x)
Instances For
A useful definition to define maps between two OneJetBundles.
Equations
Instances For
A useful definition to define maps between two OneJetBundles.
Equations
- mapLeft f Dfinv p = OneJetBundle.mk (f p.proj.1) p.proj.2 (ContinuousLinearMap.comp p.snd (Dfinv p.proj.1))
Instances For
The projection J¹(E × P, F) → J¹(E, F). Not actually used.
Instances For
The projection J¹(P × E, F) → J¹(E, F).
Equations
Instances For
In the OneJetBundle to the model space, the charts are just the canonical identification
between a product type and a bundle total space type, a.k.a. Bundle.TotalSpace.toProd.
The canonical identification between the one-jet bundle to the model space and the product, as a homeomorphism
Equations
- oneJetBundleModelSpaceHomeomorph I I' = { toEquiv := Bundle.TotalSpace.toProd (H × H') (E →L[𝕜] E'), continuous_toFun := ⋯, continuous_invFun := ⋯ }