src/HOL/Analysis/Further_Topology.thy
changeset 78131 1cadc477f644
parent 77935 7f240b0dabd9
child 78248 740b23f1138a
equal deleted inserted replaced
78130:8234c42d20e6 78131:1cadc477f644
  2682     unfolding complete_def
  2682     unfolding complete_def
  2683   proof clarify
  2683   proof clarify
  2684     fix \<sigma>
  2684     fix \<sigma>
  2685     assume \<sigma>: "\<forall>n. \<sigma> n \<in> S" and "Cauchy \<sigma>"
  2685     assume \<sigma>: "\<forall>n. \<sigma> n \<in> S" and "Cauchy \<sigma>"
  2686     have "Cauchy (f o \<sigma>)"
  2686     have "Cauchy (f o \<sigma>)"
  2687       using uniformly_continuous_imp_Cauchy_continuous \<open>Cauchy \<sigma>\<close> \<sigma> contf by blast
  2687       using uniformly_continuous_imp_Cauchy_continuous \<open>Cauchy \<sigma>\<close> \<sigma> contf
       
  2688       unfolding Cauchy_continuous_on_def by blast
  2688     then obtain l where "(f \<circ> \<sigma>) \<longlonglongrightarrow> l"
  2689     then obtain l where "(f \<circ> \<sigma>) \<longlonglongrightarrow> l"
  2689       by (auto simp: convergent_eq_Cauchy [symmetric])
  2690       by (auto simp: convergent_eq_Cauchy [symmetric])
  2690     show "\<exists>l\<in>S. \<sigma> \<longlonglongrightarrow> l"
  2691     show "\<exists>l\<in>S. \<sigma> \<longlonglongrightarrow> l"
  2691     proof
  2692     proof
  2692       show "g l \<in> S"
  2693       show "g l \<in> S"