@@ -1025,12 +1025,21 @@ theorem map_extend_nhds {x : M} (hy : x ∈ f.source) :
1025
1025
rwa [extend_coe, comp_apply, ← I.map_nhds_eq, ← f.map_nhds_eq, map_map]
1026
1026
#align local_homeomorph.map_extend_nhds PartialHomeomorph.map_extend_nhds
1027
1027
1028
+ theorem map_extend_nhds_of_boundaryless [I.Boundaryless] {x : M} (hx : x ∈ f.source) :
1029
+ map (f.extend I) (𝓝 x) = 𝓝 (f.extend I x) := by
1030
+ rw [f.map_extend_nhds _ hx, I.range_eq_univ, nhdsWithin_univ]
1031
+
1028
1032
theorem extend_target_mem_nhdsWithin {y : M} (hy : y ∈ f.source) :
1029
1033
(f.extend I).target ∈ 𝓝[range I] f.extend I y := by
1030
1034
rw [← PartialEquiv.image_source_eq_target, ← map_extend_nhds f I hy]
1031
1035
exact image_mem_map (extend_source_mem_nhds _ _ hy)
1032
1036
#align local_homeomorph.extend_target_mem_nhds_within PartialHomeomorph.extend_target_mem_nhdsWithin
1033
1037
1038
+ theorem extend_image_nhd_mem_nhds_of_boundaryless [I.Boundaryless] {x} (hx : x ∈ f.source)
1039
+ {s : Set M} (h : s ∈ 𝓝 x) : (f.extend I) '' s ∈ 𝓝 ((f.extend I) x) := by
1040
+ rw [← f.map_extend_nhds_of_boundaryless _ hx, Filter.mem_map]
1041
+ filter_upwards [h] using subset_preimage_image (f.extend I) s
1042
+
1034
1043
theorem extend_target_subset_range : (f.extend I).target ⊆ range I := by simp only [mfld_simps]
1035
1044
#align local_homeomorph.extend_target_subset_range PartialHomeomorph.extend_target_subset_range
1036
1045
@@ -1356,6 +1365,16 @@ theorem map_extChartAt_nhds : map (extChartAt I x) (𝓝 x) = 𝓝[range I] extC
1356
1365
map_extChartAt_nhds' I <| mem_extChartAt_source I x
1357
1366
#align map_ext_chart_at_nhds map_extChartAt_nhds
1358
1367
1368
+ theorem map_extChartAt_nhds_of_boundaryless [I.Boundaryless] :
1369
+ map (extChartAt I x) (𝓝 x) = 𝓝 (extChartAt I x x) := by
1370
+ rw [extChartAt]
1371
+ exact map_extend_nhds_of_boundaryless (chartAt H x) I (mem_chart_source H x)
1372
+
1373
+ theorem extChartAt_image_nhd_mem_nhds_of_boundaryless [I.Boundaryless]
1374
+ (h : s ∈ 𝓝 x) : extChartAt I x '' s ∈ 𝓝 (extChartAt I x x) := by
1375
+ rw [extChartAt]
1376
+ exact extend_image_nhd_mem_nhds_of_boundaryless _ I (mem_chart_source H x) h
1377
+
1359
1378
theorem extChartAt_target_mem_nhdsWithin' {y : M} (hy : y ∈ (extChartAt I x).source) :
1360
1379
(extChartAt I x).target ∈ 𝓝[range I] extChartAt I x y :=
1361
1380
extend_target_mem_nhdsWithin _ _ <| by rwa [← extChartAt_source I]
0 commit comments