src/HOL/Analysis/Further_Topology.thy
changeset 69745 aec42cee2521
parent 69722 b5163b2132c5
child 69922 4a9167f377b0
equal deleted inserted replaced
69744:bb0a354f6b46 69745:aec42cee2521
   653         using \<open>closed X\<close> apply blast
   653         using \<open>closed X\<close> apply blast
   654         using \<open>closed (\<Union>\<F>)\<close> apply blast
   654         using \<open>closed (\<Union>\<F>)\<close> apply blast
   655         using contf apply (force simp: elim: continuous_on_subset)
   655         using contf apply (force simp: elim: continuous_on_subset)
   656         using contg apply (force simp: elim: continuous_on_subset)
   656         using contg apply (force simp: elim: continuous_on_subset)
   657         using fh gh insert.hyps pwX by fastforce
   657         using fh gh insert.hyps pwX by fastforce
   658     then show "continuous_on (\<Union>insert X \<F> - insert a C) (\<lambda>a. if a \<in> X then f a else g a)"
   658     then show "continuous_on (\<Union>(insert X \<F>) - insert a C) (\<lambda>a. if a \<in> X then f a else g a)"
   659       by (blast intro: continuous_on_subset)
   659       by (blast intro: continuous_on_subset)
   660     show "\<forall>x\<in>(\<Union>insert X \<F> - insert a C) \<inter> K. (if x \<in> X then f x else g x) = h x"
   660     show "\<forall>x\<in>(\<Union>(insert X \<F>) - insert a C) \<inter> K. (if x \<in> X then f x else g x) = h x"
   661       using gh by (auto simp: fh)
   661       using gh by (auto simp: fh)
   662     show "(\<lambda>a. if a \<in> X then f a else g a) ` (\<Union>insert X \<F> - insert a C) \<subseteq> T"
   662     show "(\<lambda>a. if a \<in> X then f a else g a) ` (\<Union>(insert X \<F>) - insert a C) \<subseteq> T"
   663       using fim gim by auto force
   663       using fim gim by auto force
   664   qed
   664   qed
   665 qed
   665 qed
   666 
   666 
   667 
   667