src/HOL/Analysis/Abstract_Topology_2.thy
changeset 78320 eb9a9690b8f5
parent 78256 71e1aa0d9421
child 78336 6bae28577994
equal deleted inserted replaced
78284:9e0c035d026d 78320:eb9a9690b8f5
   870   proof (rule continuous_map_from_subtopology_mono)
   870   proof (rule continuous_map_from_subtopology_mono)
   871     let ?T = "{x \<in> topspace X. p x \<in> Z closure_of (topspace Z - U)}"
   871     let ?T = "{x \<in> topspace X. p x \<in> Z closure_of (topspace Z - U)}"
   872     show "continuous_map (subtopology X ?T) Y g"
   872     show "continuous_map (subtopology X ?T) Y g"
   873       by (simp add: contg)
   873       by (simp add: contg)
   874     have "X closure_of {x \<in> topspace X. p x \<notin> U} \<subseteq> X closure_of {x \<in> topspace X. p x \<in> topspace Z - U}"
   874     have "X closure_of {x \<in> topspace X. p x \<notin> U} \<subseteq> X closure_of {x \<in> topspace X. p x \<in> topspace Z - U}"
   875       by (smt (verit, del_insts) DiffI mem_Collect_eq subset_iff closure_of_mono continuous_map_closedin contp) 
   875       by (smt (verit) Collect_mono_iff DiffI closure_of_mono continuous_map contp image_subset_iff)
   876     then show "X closure_of {x \<in> topspace X. p x \<notin> U} \<subseteq> ?T"
   876     then show "X closure_of {x \<in> topspace X. p x \<notin> U} \<subseteq> ?T"
   877       by (rule order_trans [OF _ continuous_map_closure_preimage_subset [OF contp]])
   877       by (rule order_trans [OF _ continuous_map_closure_preimage_subset [OF contp]])
   878   qed
   878   qed
   879 next
   879 next
   880   show "f x = g x" if "x \<in> X frontier_of {x \<in> topspace X. p x \<in> U}" for x
   880   show "f x = g x" if "x \<in> X frontier_of {x \<in> topspace X. p x \<in> U}" for x
  1350 
  1350 
  1351 
  1351 
  1352 lemma homeomorphic_path_connected_space_imp:
  1352 lemma homeomorphic_path_connected_space_imp:
  1353      "\<lbrakk>path_connected_space X; X homeomorphic_space Y\<rbrakk> \<Longrightarrow> path_connected_space Y"
  1353      "\<lbrakk>path_connected_space X; X homeomorphic_space Y\<rbrakk> \<Longrightarrow> path_connected_space Y"
  1354   unfolding homeomorphic_space_def homeomorphic_maps_def
  1354   unfolding homeomorphic_space_def homeomorphic_maps_def
  1355   by (metis (no_types, opaque_lifting) continuous_map_closedin continuous_map_image_subset_topspace imageI order_class.order.antisym path_connectedin_continuous_map_image path_connectedin_topspace subsetI)
  1355   by (smt (verit, ccfv_threshold) homeomorphic_imp_surjective_map homeomorphic_maps_def homeomorphic_maps_map path_connectedin_continuous_map_image path_connectedin_topspace)
  1356 
  1356 
  1357 lemma homeomorphic_path_connected_space:
  1357 lemma homeomorphic_path_connected_space:
  1358    "X homeomorphic_space Y \<Longrightarrow> path_connected_space X \<longleftrightarrow> path_connected_space Y"
  1358    "X homeomorphic_space Y \<Longrightarrow> path_connected_space X \<longleftrightarrow> path_connected_space Y"
  1359   by (meson homeomorphic_path_connected_space_imp homeomorphic_space_sym)
  1359   by (meson homeomorphic_path_connected_space_imp homeomorphic_space_sym)
  1360 
  1360