src/HOL/Analysis/Abstract_Topology_2.thy
changeset 71174 7fac205dd737
parent 71172 575b3a818de5
child 71842 db120661dded
equal deleted inserted replaced
71173:caede3159e23 71174:7fac205dd737
   704       and g: "\<And>x. x \<in> topspace X \<Longrightarrow> \<exists>j. j \<in> I \<and> x \<in> T j \<and> g x = f j x"
   704       and g: "\<And>x. x \<in> topspace X \<Longrightarrow> \<exists>j. j \<in> I \<and> x \<in> T j \<and> g x = f j x"
   705     shows "continuous_map X Y g"
   705     shows "continuous_map X Y g"
   706   unfolding continuous_map_openin_preimage_eq
   706   unfolding continuous_map_openin_preimage_eq
   707 proof (intro conjI allI impI)
   707 proof (intro conjI allI impI)
   708   show "g ` topspace X \<subseteq> topspace Y"
   708   show "g ` topspace X \<subseteq> topspace Y"
   709     using g cont continuous_map_image_subset_topspace topspace_subtopology by fastforce
   709     using g cont continuous_map_image_subset_topspace by fastforce
   710 next
   710 next
   711   fix U
   711   fix U
   712   assume Y: "openin Y U"
   712   assume Y: "openin Y U"
   713   have T: "T i \<subseteq> topspace X" if "i \<in> I" for i
   713   have T: "T i \<subseteq> topspace X" if "i \<in> I" for i
   714     using ope by (simp add: openin_subset that)
   714     using ope by (simp add: openin_subset that)
   745     and g: "\<And>x. x \<in> topspace X \<Longrightarrow> \<exists>j. j \<in> I \<and> x \<in> T j \<and> g x = f j x"
   745     and g: "\<And>x. x \<in> topspace X \<Longrightarrow> \<exists>j. j \<in> I \<and> x \<in> T j \<and> g x = f j x"
   746   shows "continuous_map X Y g"
   746   shows "continuous_map X Y g"
   747   unfolding continuous_map_closedin_preimage_eq
   747   unfolding continuous_map_closedin_preimage_eq
   748 proof (intro conjI allI impI)
   748 proof (intro conjI allI impI)
   749   show "g ` topspace X \<subseteq> topspace Y"
   749   show "g ` topspace X \<subseteq> topspace Y"
   750     using g cont continuous_map_image_subset_topspace topspace_subtopology by fastforce
   750     using g cont continuous_map_image_subset_topspace by fastforce
   751 next
   751 next
   752   fix U
   752   fix U
   753   assume Y: "closedin Y U"
   753   assume Y: "closedin Y U"
   754   have T: "T i \<subseteq> topspace X" if "i \<in> I" for i
   754   have T: "T i \<subseteq> topspace X" if "i \<in> I" for i
   755     using clo by (simp add: closedin_subset that)
   755     using clo by (simp add: closedin_subset that)