@@ -807,24 +807,6 @@ theorem mem_analyticGroupoid_of_boundaryless [CompleteSpace E] [I.Boundaryless]
807
807
808
808
end analyticGroupoid
809
809
810
- /-! Topological manifolds with corners: no smoothness assumed, but boundary and/or corners
811
- are possible. -/
812
- section ManifoldWithCorners
813
- /-- Typeclass defining topological manifolds with corners with respect to a model with corners,
814
- over a field `π`. -/
815
- class ManifoldWithCorners {π : Type *} [NontriviallyNormedField π] {E : Type *}
816
- [NormedAddCommGroup E] [NormedSpace π E] {H : Type *} [TopologicalSpace H]
817
- (I : ModelWithCorners π E H) (M : Type *) [TopologicalSpace M] [ChartedSpace H M] extends
818
- HasGroupoid M (contDiffGroupoid 0 I) : Prop
819
-
820
- theorem ManifoldWithCorners.mk' {π : Type *} [NontriviallyNormedField π] {E : Type *}
821
- [NormedAddCommGroup E] [NormedSpace π E] {H : Type *} [TopologicalSpace H]
822
- (I : ModelWithCorners π E H) (M : Type *) [TopologicalSpace M] [ChartedSpace H M]
823
- [gr : HasGroupoid M (contDiffGroupoid 0 I)] : ManifoldWithCorners I M :=
824
- { gr with }
825
-
826
- end ManifoldWithCorners
827
-
828
810
section SmoothManifoldWithCorners
829
811
830
812
/-! ### Smooth manifolds with corners -/
@@ -1006,9 +988,6 @@ theorem mapsTo_extend (hs : s β f.source) :
1006
988
exact image_subset _ (inter_subset_right _ _)
1007
989
#align local_homeomorph.maps_to_extend LocalHomeomorph.mapsTo_extend
1008
990
1009
- lemma mapsTo_extend' : MapsTo (f.extend I) (f.extend I).source (f.extend I).target :=
1010
- fun _ hx β¦(f.extend I).map_source hx
1011
-
1012
991
theorem extend_left_inv {x : M} (hxf : x β f.source) : (f.extend I).symm (f.extend I x) = x :=
1013
992
(f.extend I).left_inv <| by rwa [f.extend_source]
1014
993
#align local_homeomorph.extend_left_inv LocalHomeomorph.extend_left_inv
0 commit comments