Documentation

Mathlib.Geometry.Manifold.MFDeriv.Tangent

Derivatives of maps in the tangent bundle #

This file contains properties of derivatives which need the manifold structure of the tangent bundle. Notably, it includes formulas for the tangent maps to charts, and unique differentiability statements for subsets of the tangent bundle.

theorem tangentMap_chart {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} [NormedAddCommGroup E] [NormedSpace ๐•œ E] {H : Type u_3} [TopologicalSpace H] {I : ModelWithCorners ๐•œ E H} {M : Type u_4} [TopologicalSpace M] [ChartedSpace H M] [SmoothManifoldWithCorners I M] {p : TangentBundle I M} {q : TangentBundle I M} (h : q.proj โˆˆ (chartAt H p.proj).source) :
tangentMap I I (โ†‘(chartAt H p.proj)) q = (Bundle.TotalSpace.toProd H E).symm (โ†‘(chartAt (ModelProd H E) p) q)

The derivative of the chart at a base point is the chart of the tangent bundle, composed with the identification between the tangent bundle of the model space and the product space.

theorem tangentMap_chart_symm {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} [NormedAddCommGroup E] [NormedSpace ๐•œ E] {H : Type u_3} [TopologicalSpace H] {I : ModelWithCorners ๐•œ E H} {M : Type u_4} [TopologicalSpace M] [ChartedSpace H M] [SmoothManifoldWithCorners I M] {p : TangentBundle I M} {q : TangentBundle I H} (h : q.proj โˆˆ (chartAt H p.proj).target) :
tangentMap I I (โ†‘(chartAt H p.proj).symm) q = โ†‘(chartAt (ModelProd H E) p).symm ((Bundle.TotalSpace.toProd H E) q)

The derivative of the inverse of the chart at a base point is the inverse of the chart of the tangent bundle, composed with the identification between the tangent bundle of the model space and the product space.

theorem mfderiv_chartAt_eq_tangentCoordChange {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} [NormedAddCommGroup E] [NormedSpace ๐•œ E] {H : Type u_3} [TopologicalSpace H] {I : ModelWithCorners ๐•œ E H} {M : Type u_4} [TopologicalSpace M] [ChartedSpace H M] [SmoothManifoldWithCorners I M] {x : M} {y : M} (hsrc : x โˆˆ (chartAt H y).source) :
mfderiv I I (โ†‘(chartAt H y)) x = tangentCoordChange I x y x
theorem UniqueMDiffOn.tangentBundle_proj_preimage {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} [NormedAddCommGroup E] [NormedSpace ๐•œ E] {H : Type u_3} [TopologicalSpace H] {I : ModelWithCorners ๐•œ E H} {M : Type u_4} [TopologicalSpace M] [ChartedSpace H M] [SmoothManifoldWithCorners I M] {s : Set M} (hs : UniqueMDiffOn I s) :
UniqueMDiffOn I.tangent (Bundle.TotalSpace.proj โปยน' s)

The preimage under the projection from the tangent bundle of a set with unique differential in the basis also has unique differential.