src/HOL/Multivariate_Analysis/Topology_Euclidean_Space.thy
changeset 44138 0c9feac80852
parent 44133 691c52e900ca
child 44139 abccf1b7ea4b
equal deleted inserted replaced
44137:ac5cb4c86448 44138:0c9feac80852
  2226     using compact_real_lemma [OF b] by auto
  2226     using compact_real_lemma [OF b] by auto
  2227   thus "\<exists>l r. subseq r \<and> ((f \<circ> r) ---> l) sequentially"
  2227   thus "\<exists>l r. subseq r \<and> ((f \<circ> r) ---> l) sequentially"
  2228     by auto
  2228     by auto
  2229 qed
  2229 qed
  2230 
  2230 
  2231 lemma bounded_component: "bounded s \<Longrightarrow>
  2231 lemma bounded_component: "bounded s \<Longrightarrow> bounded ((\<lambda>x. x $$ i) ` s)"
  2232   bounded ((\<lambda>x. x $$ i) ` (s::'a::euclidean_space set))"
  2232   apply (erule bounded_linear_image)
  2233 unfolding bounded_def
  2233   apply (rule bounded_linear_euclidean_component)
  2234 apply clarify
  2234   done
  2235 apply (rule_tac x="x $$ i" in exI)
       
  2236 apply (rule_tac x="e" in exI)
       
  2237 apply clarify
       
  2238 apply (rule order_trans[OF dist_nth_le],simp)
       
  2239 done
       
  2240 
  2235 
  2241 lemma compact_lemma:
  2236 lemma compact_lemma:
  2242   fixes f :: "nat \<Rightarrow> 'a::euclidean_space"
  2237   fixes f :: "nat \<Rightarrow> 'a::euclidean_space"
  2243   assumes "bounded s" and "\<forall>n. f n \<in> s"
  2238   assumes "bounded s" and "\<forall>n. f n \<in> s"
  2244   shows "\<forall>d. \<exists>l::'a. \<exists> r. subseq r \<and>
  2239   shows "\<forall>d. \<exists>l::'a. \<exists> r. subseq r \<and>