Documentation

Mathlib.Geometry.Manifold.AnalyticManifold

Analytic manifolds (possibly with boundary or corners) #

An analytic manifold is a manifold modelled on a normed vector space, or a subset like a half-space (to get manifolds with boundaries) for which changes of coordinates are analytic in the interior and smooth everywhere (including at the boundary). The definition mirrors SmoothManifoldWithCorners, but using an analyticGroupoid in place of contDiffGroupoid. All analytic manifolds are smooth manifolds.

Completeness is required throughout, but this is nonessential: it is due to many of the lemmas about AnalyticWithinOn` requiring completeness for ease of proof.

analyticGroupoid #

f โˆˆ PartialHomeomorph H H is in analyticGroupoid I if f and f.symm are smooth everywhere, analytic on the interior, and map the interior to itself. This allows us to define AnalyticManifold including in cases with boundary.

def analyticPregroupoid {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [CompleteSpace E] {H : Type u_3} [TopologicalSpace H] (I : ModelWithCorners ๐•œ E H) :

Given a model with corners (E, H), we define the pregroupoid of analytic transformations of H as the maps that are AnalyticWithinOn when read in E through I. Using AnalyticWithinOn rather than AnalyticOn gives us meaningful definitions at boundary points.

Equations
Instances For
    def analyticGroupoid {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [CompleteSpace E] {H : Type u_3} [TopologicalSpace H] (I : ModelWithCorners ๐•œ E H) :

    Given a model with corners (E, H), we define the groupoid of analytic transformations of H as the maps that are AnalyticWithinOn when read in E through I. Using AnalyticWithinOn rather than AnalyticOn gives us meaningful definitions at boundary points.

    Equations
    Instances For
      theorem ofSet_mem_analyticGroupoid {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [CompleteSpace E] {H : Type u_3} [TopologicalSpace H] (I : ModelWithCorners ๐•œ E H) {s : Set H} (hs : IsOpen s) :

      An identity partial homeomorphism belongs to the analytic groupoid.

      theorem symm_trans_mem_analyticGroupoid {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [CompleteSpace E] {H : Type u_3} [TopologicalSpace H] (I : ModelWithCorners ๐•œ E H) {M : Type u_4} [TopologicalSpace M] (e : PartialHomeomorph M H) :
      e.symm.trans e โˆˆ analyticGroupoid I

      The composition of a partial homeomorphism from H to M and its inverse belongs to the analytic groupoid.

      The analytic groupoid is closed under restriction.

      Equations
      • โ‹ฏ = โ‹ฏ
      theorem mem_analyticGroupoid {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [CompleteSpace E] {H : Type u_3} [TopologicalSpace H] {I : ModelWithCorners ๐•œ E H} {f : PartialHomeomorph H H} :
      f โˆˆ analyticGroupoid I โ†” AnalyticWithinOn ๐•œ (โ†‘I โˆ˜ โ†‘f โˆ˜ โ†‘I.symm) (โ†‘I.symm โปยน' f.source โˆฉ Set.range โ†‘I) โˆง AnalyticWithinOn ๐•œ (โ†‘I โˆ˜ โ†‘f.symm โˆ˜ โ†‘I.symm) (โ†‘I.symm โปยน' f.target โˆฉ Set.range โ†‘I)

      f โˆˆ analyticGroupoid iff it and its inverse are analytic within range I.

      theorem mem_analyticGroupoid_of_boundaryless {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [CompleteSpace E] {H : Type u_3} [TopologicalSpace H] (I : ModelWithCorners ๐•œ E H) [I.Boundaryless] (e : PartialHomeomorph H H) :
      e โˆˆ analyticGroupoid I โ†” AnalyticOn ๐•œ (โ†‘I โˆ˜ โ†‘e โˆ˜ โ†‘I.symm) (โ†‘I '' e.source) โˆง AnalyticOn ๐•œ (โ†‘I โˆ˜ โ†‘e.symm โˆ˜ โ†‘I.symm) (โ†‘I '' e.target)

      The analytic groupoid on a boundaryless charted space modeled on a complete vector space consists of the partial homeomorphisms which are analytic and have analytic inverse.

      theorem analyticGroupoid_prod {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type} {A : Type} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [CompleteSpace E] [TopologicalSpace A] {F : Type} {B : Type} [NormedAddCommGroup F] [NormedSpace ๐•œ F] [CompleteSpace F] [TopologicalSpace B] {I : ModelWithCorners ๐•œ E A} {J : ModelWithCorners ๐•œ F B} {f : PartialHomeomorph A A} {g : PartialHomeomorph B B} (fa : f โˆˆ analyticGroupoid I) (ga : g โˆˆ analyticGroupoid J) :
      f.prod g โˆˆ analyticGroupoid (I.prod J)

      analyticGroupoid is closed under products

      class AnalyticManifold {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [CompleteSpace E] {H : Type u_3} [TopologicalSpace H] (I : ModelWithCorners ๐•œ E H) (M : Type u_5) [TopologicalSpace M] [ChartedSpace H M] extends HasGroupoid :

      An analytic manifold w.r.t. a model I : ModelWithCorners ๐•œ E H is a charted space over H s.t. all extended chart conversion maps are analytic.

        Instances
          instance AnalyticManifold.self {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [CompleteSpace E] :

          Normed spaces are analytic manifolds over themselves.

          Equations
          • โ‹ฏ = โ‹ฏ
          instance AnalyticManifold.prod {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type} {A : Type} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [CompleteSpace E] [TopologicalSpace A] {F : Type} {B : Type} [NormedAddCommGroup F] [NormedSpace ๐•œ F] [CompleteSpace F] [TopologicalSpace B] {I : ModelWithCorners ๐•œ E A} {J : ModelWithCorners ๐•œ F B} {M : Type} [TopologicalSpace M] [ChartedSpace A M] [m : AnalyticManifold I M] {N : Type} [TopologicalSpace N] [ChartedSpace B N] [n : AnalyticManifold J N] :
          AnalyticManifold (I.prod J) (M ร— N)

          M ร— N is an analytic manifold if M and N are

          Equations
          • โ‹ฏ = โ‹ฏ
          instance AnalyticManifold.smoothManifoldWithCorners {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [CompleteSpace E] {H : Type u_3} [TopologicalSpace H] (I : ModelWithCorners ๐•œ E H) {M : Type u_4} [TopologicalSpace M] [ChartedSpace H M] [cm : AnalyticManifold I M] :

          Analytic manifolds are smooth manifolds.

          Equations
          • โ‹ฏ = โ‹ฏ