Documentation

Mathlib.Geometry.Manifold.Instances.Icc

Manifold structure on real intervals #

The manifold structure on real intervals is defined in Mathlib.Geometry.Manifold.Instances.Real. We relate it to the manifold structure on the real line, by showing that the inclusion (contMDiff_subtype_coe_Icc) and projection (contMDiffOn_projIcc) are smooth, and showing that a function defined on the interval is smooth iff its composition with the projection is smooth on the interval in โ„ (see contMDiffOn_comp_projIcc_iff and friends).

We also define 1 : TangentSpace (๐“กโˆ‚ 1) z, and relate it to 1 in the real line.

TODO #

This file can be thoroughly rewritten once mathlib has a good theory of smooth immersions and embeddings. Once this is done,

@[irreducible]
def oneTangentSpaceIcc {x y : โ„} [h : Fact (x < y)] (z : โ†‘(Set.Icc x y)) :

Unit vector in the tangent space to a segment, as the image of the unit vector in the real line under the canonical projection. It is also mapped to the unit vector in the real line through the canonical injection, see mfderiv_subtype_coe_Icc_one.

Note that one can not abuse defeqs for this definition: this is not the same as the vector fun _ โ†ฆ 1 in EuclideanSpace โ„ (Fin 1) through defeqs, as one of the charts of Icc x y is orientation-reversing.

Equations
Instances For

    The inclusion map from of a closed segment to โ„ is smooth in the manifold sense.

    The projection from โ„ to a closed segment is smooth on the segment, in the manifold sense.

    theorem contMDiffWithinAt_comp_projIcc_iff {E : Type u_1} [NormedAddCommGroup E] [NormedSpace โ„ E] {H : Type u_2} [TopologicalSpace H] {I : ModelWithCorners โ„ E H} {M : Type u_3} [TopologicalSpace M] [ChartedSpace H M] {x y : โ„} [h : Fact (x < y)] {n : WithTop โ„•โˆž} {f : โ†‘(Set.Icc x y) โ†’ M} {w : โ†‘(Set.Icc x y)} :
    theorem mfderivWithin_comp_projIcc_one {E : Type u_1} [NormedAddCommGroup E] [NormedSpace โ„ E] {H : Type u_2} [TopologicalSpace H] {I : ModelWithCorners โ„ E H} {M : Type u_3} [TopologicalSpace M] [ChartedSpace H M] {x y : โ„} [h : Fact (x < y)] {f : โ†‘(Set.Icc x y) โ†’ M} {w : โ†‘(Set.Icc x y)} :