src/HOL/Analysis/Function_Topology.thy
changeset 64845 e5d4bc2016a6
parent 64289 42f28160bad9
child 64910 6108dddad9f0
equal deleted inserted replaced
64844:bb70dc05cd38 64845:e5d4bc2016a6
   290   then have "g x \<in> f-`(topspace T2)"
   290   then have "g x \<in> f-`(topspace T2)"
   291     unfolding comp_def by blast
   291     unfolding comp_def by blast
   292   moreover have "g x \<in> A" using assms(2) `x \<in> topspace T1` by blast
   292   moreover have "g x \<in> A" using assms(2) `x \<in> topspace T1` by blast
   293   ultimately show "g x \<in> topspace (pullback_topology A f T2)"
   293   ultimately show "g x \<in> topspace (pullback_topology A f T2)"
   294     unfolding topspace_pullback_topology by blast
   294     unfolding topspace_pullback_topology by blast
   295 qed
       
   296 
       
   297 subsubsection {*Miscellaneous*}
       
   298 
       
   299 text {*The following could belong to \verb+Topology_Euclidean_Spaces.thy+, and will be needed
       
   300 below.*}
       
   301 lemma openin_INT [intro]:
       
   302   assumes "finite I"
       
   303           "\<And>i. i \<in> I \<Longrightarrow> openin T (U i)"
       
   304   shows "openin T ((\<Inter>i \<in> I. U i) \<inter> topspace T)"
       
   305 using assms by (induct, auto simp add: inf_sup_aci(2) openin_Int)
       
   306 
       
   307 lemma openin_INT2 [intro]:
       
   308   assumes "finite I" "I \<noteq> {}"
       
   309           "\<And>i. i \<in> I \<Longrightarrow> openin T (U i)"
       
   310   shows "openin T (\<Inter>i \<in> I. U i)"
       
   311 proof -
       
   312   have "(\<Inter>i \<in> I. U i) \<subseteq> topspace T"
       
   313     using `I \<noteq> {}` openin_subset[OF assms(3)] by auto
       
   314   then show ?thesis
       
   315     using openin_INT[of _ _ U, OF assms(1) assms(3)] by (simp add: inf.absorb2 inf_commute)
       
   316 qed
   295 qed
   317 
   296 
   318 
   297 
   319 subsection {*The product topology*}
   298 subsection {*The product topology*}
   320 
   299