Sections of 1-jet bundles #
In this file we study sections of 1-jet bundles. This is the direct continuation
of OneJetBundle.lean
but it imports more files, hence the cut.
Main definitions #
In this file we consider two manifolds M
and M'
with models I
and I'
OneJetSet I M I' M'
: smooth sections ofOneJetBundle I M I' M' → M
A section of a 1-jet bundle seen as a bundle over the source manifold.
- bs : M → M'
- smooth' : ContMDiff I ((I.prod I').prod (modelWithCornersSelf 𝕜 (E →L[𝕜] E'))) ↑⊤ fun (x : M) => OneJetBundle.mk x (self.bs x) (self.ϕ x)
Instances For
Equations
- instFunLikeOneJetSecOneJetBundle I M I' M' = { coe := fun (S : OneJetSec I M I' M') (x : M) => OneJetBundle.mk x (S.bs x) (S.ϕ x), coe_injective' := ⋯ }
Equations
- OneJetSec.mk' F hF h2F = { bs := fun (x : M) => (F x).proj.2, ϕ := fun (x : M) => (F x).snd, smooth' := ⋯ }
Instances For
A section of J¹(M, M') is holonomic at (x : M) if its linear map part is the derivative of its base map at x.
Instances For
A section of J¹(M, M') is holonomic at (x : M) iff it coincides with the 1-jet extension of its base map at x.
A map from M to J¹(M, M') is holonomic if its linear map part is the derivative of its base map at every point.
Equations
- F.IsHolonomic = ∀ (x : M), F.IsHolonomicAt x
Instances For
Equations
- IsHolonomicGerm φ = Quotient.liftOn' φ (fun (F : M → OneJetBundle I M I' M') => mfderiv I I' (fun (x' : M) => (F x').proj.2) x = (F x).snd) ⋯
Instances For
The one-jet extension of a function, seen as a section of the 1-jet bundle.
Equations
- oneJetExtSec f = { bs := ⇑f, ϕ := mfderiv I I' ⇑f, smooth' := ⋯ }
Instances For
A family of jet sections indexed by manifold N
is a function from N
into jet sections
in such a way that the function is smooth as a function of all arguments.
- bs : N → M → M'
Instances For
Equations
- instFunLikeFamilyOneJetSecOneJetSecReal I M I' M' J N = { coe := fun (S : FamilyOneJetSec I M I' M' J N) (t : N) => { bs := S.bs t, ϕ := S.ϕ t, smooth' := ⋯ }, coe_injective' := ⋯ }
Equations
- FamilyOneJetSec.mk' FF hF h2F = { bs := fun (s : N) (x : M) => (FF s x).proj.2, ϕ := fun (s : N) (x : M) => (FF s x).snd, smooth' := ⋯ }
Instances For
Reindex a family along a smooth function f
.
Equations
Instances For
Turn a family of sections of J¹(M, M')
parametrized by N
into a section of J¹(N × M, M')
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
A homotopy of 1-jet sections is a family of 1-jet sections indexed by ℝ
Equations
- HtpyOneJetSec I M I' M' = FamilyOneJetSec I M I' M' (modelWithCornersSelf ℝ ℝ) ℝ