src/HOL/Multivariate_Analysis/Topology_Euclidean_Space.thy
changeset 46887 cb891d9a23c1
parent 45776 714100f5fda4
child 47108 2a1953f0d20d
equal deleted inserted replaced
46886:4cd29473c65d 46887:cb891d9a23c1
  3173     with `?lhs` obtain d where "d>0" and d:"\<forall>x\<in>s. 0 < dist x a \<and> dist x a < d \<longrightarrow> f x \<in> T"
  3173     with `?lhs` obtain d where "d>0" and d:"\<forall>x\<in>s. 0 < dist x a \<and> dist x a < d \<longrightarrow> f x \<in> T"
  3174       unfolding continuous_within tendsto_def eventually_within by auto
  3174       unfolding continuous_within tendsto_def eventually_within by auto
  3175     have "eventually (\<lambda>n. dist (x n) a < d) sequentially"
  3175     have "eventually (\<lambda>n. dist (x n) a < d) sequentially"
  3176       using x(2) `d>0` by simp
  3176       using x(2) `d>0` by simp
  3177     hence "eventually (\<lambda>n. (f \<circ> x) n \<in> T) sequentially"
  3177     hence "eventually (\<lambda>n. (f \<circ> x) n \<in> T) sequentially"
  3178     proof (rule eventually_elim1)
  3178     proof eventually_elim
  3179       fix n assume "dist (x n) a < d" thus "(f \<circ> x) n \<in> T"
  3179       case (elim n) thus ?case
  3180         using d x(1) `f a \<in> T` unfolding dist_nz[THEN sym] by auto
  3180         using d x(1) `f a \<in> T` unfolding dist_nz[THEN sym] by auto
  3181     qed
  3181     qed
  3182   }
  3182   }
  3183   thus ?rhs unfolding tendsto_iff unfolding tendsto_def by simp
  3183   thus ?rhs unfolding tendsto_iff unfolding tendsto_def by simp
  3184 next
  3184 next