Manifold structure on the sphere #
This file defines stereographic projection from the sphere in an inner product space E, and uses it to put an analytic manifold structure on the sphere.
Main results #
For a unit vector v in E, the definition stereographic gives the stereographic projection centred at v, an open partial homeomorphism from the sphere to (ℝ ∙ v)ᗮ (the orthogonal complement of v).
For finite-dimensional E, we then construct an analytic manifold instance on the sphere; the charts here are obtained by composing the open partial homeomorphisms stereographic with arbitrary isometries from (ℝ ∙ v)ᗮ to Euclidean space.
We prove two lemmas about C^n maps:
contMDiff_coe_spherestates that the coercion map from the sphere intoEis analytic; this is a useful tool for constructing smooth maps from the sphere.contMDiff.codRestrict_spherestates that a map from a manifold into the sphere isC^mif its lift to a map toEisC^m; this is a useful tool for constructingC^mmaps to the sphere.
As an application we prove contMDiffNegSphere, that the antipodal map is analytic.
Finally, we equip the Circle (defined in Analysis.Complex.Circle to be the sphere in ℂ centred at 0 of radius 1) with the following structure:
- a charted space with model space
EuclideanSpace ℝ (Fin 1)(inherited fromMetric.Sphere) - an analytic Lie group with model with corners
𝓡 1
We furthermore show that Circle.exp (defined in Analysis.Complex.Circle to be the natural map fun t ↦ exp (t * I) from ℝ to Circle) is analytic.
Implementation notes #
The model space for the charted space instance is EuclideanSpace ℝ (Fin n), where n is a natural number satisfying the typeclass assumption [Fact (finrank ℝ E = n + 1)]. This may seem a little awkward, but it is designed to circumvent the problem that the literal expression for the dimension of the model space (up to definitional equality) determines the type. If one used the naive expression EuclideanSpace ℝ (Fin (finrank ℝ E - 1)) for the model space, then the sphere in ℂ would be a manifold with model space EuclideanSpace ℝ (Fin (2 - 1)) but not with model space EuclideanSpace ℝ (Fin 1).
TODO #
Relate the stereographic projection to the inversion of the space.
Construction of the stereographic projection #
Stereographic projection, forward direction. This is a map from an inner product space E to the orthogonal complement of an element v of E. It is smooth away from the affine hyperplane through v parallel to the orthogonal complement. It restricts on the sphere to the stereographic projection.
Instances For
Auxiliary function for the construction of the reverse direction of the stereographic projection. This is a map from the orthogonal complement of a unit vector v in an inner product space E to E; we will later prove that it takes values in the unit sphere.
For most purposes, use stereoInvFun, not stereoInvFunAux.
Instances For
Stereographic projection, reverse direction. This is a map from the orthogonal complement of a unit vector v in an inner product space E to the unit sphere in E.
Equations
- stereoInvFun hv w = ⟨stereoInvFunAux v ↑w, ⋯⟩
Instances For
Stereographic projection from the unit sphere in E, centred at a unit vector v in E; this is the version as an open partial homeomorphism.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Charted space structure on the sphere #
In this section we construct a charted space structure on the unit sphere in a finite-dimensional real inner product space E; that is, we show that it is locally homeomorphic to the Euclidean space of dimension one less than E.
The restriction to finite dimension is for convenience. The most natural ChartedSpace structure for the sphere uses the stereographic projection from the antipodes of a point as the canonical chart at this point. However, the codomain of the stereographic projection constructed in the previous section is (ℝ ∙ v)ᗮ, the orthogonal complement of the vector v in E which is the "north pole" of the projection, so a priori these charts all have different codomains.
So it is necessary to prove that these codomains are all continuously linearly equivalent to a fixed normed space. This could be proved in general by a simple case of Gram-Schmidt orthogonalization, but in the finite-dimensional case it follows more easily by dimension-counting.
Variant of the stereographic projection, for the sphere in an n + 1-dimensional inner product space E. This version has codomain the Euclidean space of dimension n, and is obtained by composing the original stereographic projection (stereographic) with an arbitrary linear isometry from (ℝ ∙ v)ᗮ to the Euclidean space.
Equations
Instances For
The unit sphere in an n + 1-dimensional inner product space E is a charted space modelled on the Euclidean space of dimension n.
Equations
- One or more equations did not get rendered due to their size.
Analytic manifold structure on the sphere #
The unit sphere in an n + 1-dimensional inner product space E is an analytic manifold, modelled on the Euclidean space of dimension n.
The inclusion map (i.e., coe) from the sphere in E to E is analytic.
If a C^m function f : M → E, where M is some manifold, takes values in the sphere, then it restricts to a C^m function from M to the sphere.
The antipodal map is analytic.
Consider the differential of the inclusion of the sphere in E at the point v as a continuous linear map from TangentSpace (𝓡 n) v to E. The range of this map is the orthogonal complement of v in E.
Note that there is an abuse here of the defeq between E and the tangent space to E at (v:E). In general this defeq is not canonical, but in this case (the tangent space of a vector space) it is canonical.
Consider the differential of the inclusion of the sphere in E at the point v as a continuous linear map from TangentSpace (𝓡 n) v to E. This map is injective.
Local instance to help the typeclass system to figure out 1 + 1 = 2.
The unit circle in ℂ is a charted space modelled on EuclideanSpace ℝ (Fin 1). This follows by definition from the corresponding result for Metric.Sphere.
The unit circle in ℂ is an analytic Lie group.
The map fun t ↦ exp (t * I) from ℝ to the unit circle in ℂ is analytic.