Documentation

Orbifolds.Diffeology.Manifolds

Diffeological manifolds #

Some lemmas and theorems on manifolds as diffeological spaces, as defined in Orbifolds.Diffeology.LocallyModelled. The main purpose of this file is to show how this relates to the notion of smooth manifolds defined in mathlib , i.e. that those are indeed equivalent.

The diffeology defined by a manifold structure on M, with the plots given by the maps that are smooth in the sense of mathlib's ContMDiff-API. This can not be an instance because IsManifold I M depends on I while DiffeologicalSpace M does not, and because it would probably lead to instance diamonds on things like products even if some workaround was found.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    theorem isPlot_iff_contMDiff {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] [m : IsManifold I (↑) M] {n : } {p : Eucl nM} :

    The plots of a manifold are by definition precisely the smooth maps.

    Equations
    • I.toHomeomorphTarget = { toFun := fun (x : H) => I x, , invFun := fun (y : I.target) => I.invFun y, left_inv := , right_inv := , continuous_toFun := , continuous_invFun := }
    Instances For
      theorem IsManifold.dTop_le {E : Type u_1} [NormedAddCommGroup E] [NormedSpace E] {H : Type u_2} [TopologicalSpace H] (I : ModelWithCorners E H) (M : Type u_3) [tM : TopologicalSpace M] [ChartedSpace H M] [m : IsManifold I (↑) M] :

      The D-topology on a manifold is always at least as fine as the usual topology.

      theorem ContMDiff.dsmooth {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] [m : IsManifold I (↑) M] {E' : Type u_4} [NormedAddCommGroup E'] [NormedSpace E'] {H' : Type u_5} [TopologicalSpace H'] {I' : ModelWithCorners E' H'} {N : Type u_6} [TopologicalSpace N] [ChartedSpace H' N] [m' : IsManifold I' (↑) N] {f : MN} (hf : ContMDiff I I' (↑) f) :

      Every smooth map between manifolds is also D-smooth, i.e. this construction defines a functor of concrete categories.

      theorem ContMDiffOn.dsmooth_restrict {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] [m : IsManifold I (↑) M] {E' : Type u_4} [NormedAddCommGroup E'] [NormedSpace E'] {H' : Type u_5} [TopologicalSpace H'] {I' : ModelWithCorners E' H'} {N : Type u_6} [TopologicalSpace N] [ChartedSpace H' N] [m' : IsManifold I' (↑) N] {f : MN} {s : Set M} (hf : ContMDiffOn I I' (↑) f s) :

      Every map between manifolds that is smooth on a subset is also smooth diffeologically with respect to the subspace diffeology.

      theorem IsOpen.dsmooth_iff_smoothOn {E : Type u_1} [NormedAddCommGroup E] [NormedSpace E] [FiniteDimensional E] {H : Type u_2} [TopologicalSpace H] {I : ModelWithCorners E H} (M : Type u_3) [TopologicalSpace M] [ChartedSpace H M] [m : IsManifold I (↑) M] [hI : I.Boundaryless] {E' : Type u_4} [NormedAddCommGroup E'] [NormedSpace E'] [FiniteDimensional E'] {H' : Type u_5} [TopologicalSpace H'] {I' : ModelWithCorners E' H'} (N : Type u_6) [TopologicalSpace N] [ChartedSpace H' N] [m' : IsManifold I' (↑) N] {f : MN} {s : Set M} (hs : IsOpen s) :
      let x := IsManifold.toDiffeology I M; let x_1 := IsManifold.toDiffeology I' N; DSmooth (s.restrict f) ContMDiffOn I I' (↑) f s

      Every D-smooth map from a boundaryless manifold to another manifold is also smooth. This could probably be proven in quite a lot greater generality.

      theorem DSmooth.smooth {E : Type u_1} [NormedAddCommGroup E] [NormedSpace E] [FiniteDimensional E] {H : Type u_2} [TopologicalSpace H] {I : ModelWithCorners E H} {M : Type u_3} [TopologicalSpace M] [ChartedSpace H M] [m : IsManifold I (↑) M] [hI : I.Boundaryless] {E' : Type u_4} [NormedAddCommGroup E'] [NormedSpace E'] [FiniteDimensional E'] {H' : Type u_5} [TopologicalSpace H'] {I' : ModelWithCorners E' H'} {N : Type u_6} [TopologicalSpace N] [ChartedSpace H' N] [m' : IsManifold I' (↑) N] {f : MN} (hf : DSmooth f) :
      ContMDiff I I' (↑) f

      Every D-smooth map from a boundaryless manifold to another manifold is also smooth. This could probably be proven in quite a lot greater generality.

      A finite-dimensional, boundaryless smooth manifold with corners in the sense of IsManifold is also a manifold in the sense of IsDiffeologicalManifold.

      noncomputable def PartialEquiv.fromEquivSourceTarget {α : Type u_1} {β : Type u_2} {s : Set α} {t : Set β} (e : s t) (a : s) :
      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        @[simp]
        theorem PartialEquiv.fromEquivSourceTarget_target {α : Type u_1} {β : Type u_2} {s : Set α} {t : Set β} (e : s t) (a : s) :
        @[simp]
        theorem PartialEquiv.fromEquivSourceTarget_symm_apply {α : Type u_1} {β : Type u_2} {s : Set α} {t : Set β} (e : s t) (a : s) (y : β) :
        (fromEquivSourceTarget e a).symm y = if hy : y t then (e.symm y, hy) else a
        @[simp]
        theorem PartialEquiv.fromEquivSourceTarget_source {α : Type u_1} {β : Type u_2} {s : Set α} {t : Set β} (e : s t) (a : s) :
        @[simp]
        theorem PartialEquiv.fromEquivSourceTarget_apply {α : Type u_1} {β : Type u_2} {s : Set α} {t : Set β} (e : s t) (a : s) (x : α) :
        (fromEquivSourceTarget e a) x = if hx : x s then (e x, hx) else (e a)
        @[simp]
        theorem PartialEquiv.fromEquivSourceTarget_restrict {α : Type u_1} {β : Type u_2} {s : Set α} {t : Set β} (e : s t) (a : s) :
        @[simp]
        theorem PartialEquiv.fromEquivSourceTarget_symm_restrict {α : Type u_1} {β : Type u_2} {s : Set α} {t : Set β} (e : s t) (a : s) :
        @[simp]
        theorem PartialEquiv.fromEquivSourceTarget_toEquiv {α : Type u_1} {β : Type u_2} {s : Set α} {t : Set β} (e : s t) (a : s) :
        noncomputable def PartialHomeomorph.fromHomeomorphSourceTarget {α : Type u_1} {β : Type u_2} [TopologicalSpace α] [TopologicalSpace β] {s : Set α} {t : Set β} (e : s ≃ₜ t) (hs : IsOpen s) (ht : IsOpen t) (a : s) :
        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          @[simp]
          theorem PartialHomeomorph.fromHomeomorphSourceTarget_symm_apply {α : Type u_1} {β : Type u_2} [TopologicalSpace α] [TopologicalSpace β] {s : Set α} {t : Set β} (e : s ≃ₜ t) (hs : IsOpen s) (ht : IsOpen t) (a : s) (y : β) :
          (fromHomeomorphSourceTarget e hs ht a).symm y = if hy : y t then (e.symm y, hy) else a
          @[simp]
          theorem PartialHomeomorph.fromHomeomorphSourceTarget_target {α : Type u_1} {β : Type u_2} [TopologicalSpace α] [TopologicalSpace β] {s : Set α} {t : Set β} (e : s ≃ₜ t) (hs : IsOpen s) (ht : IsOpen t) (a : s) :
          @[simp]
          theorem PartialHomeomorph.fromHomeomorphSourceTarget_apply {α : Type u_1} {β : Type u_2} [TopologicalSpace α] [TopologicalSpace β] {s : Set α} {t : Set β} (e : s ≃ₜ t) (hs : IsOpen s) (ht : IsOpen t) (a : s) (x : α) :
          (fromHomeomorphSourceTarget e hs ht a) x = if hx : x s then (e x, hx) else (e a)
          @[simp]
          theorem PartialHomeomorph.fromHomeomorphSourceTarget_source {α : Type u_1} {β : Type u_2} [TopologicalSpace α] [TopologicalSpace β] {s : Set α} {t : Set β} (e : s ≃ₜ t) (hs : IsOpen s) (ht : IsOpen t) (a : s) :
          @[simp]

          Charted space structure of a diffeological manifold, consisting of all local diffeomorphisms between M and Eucl n.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For