src/HOL/Multivariate_Analysis/Finite_Cartesian_Product.thy
changeset 50880 b22ecedde1c7
parent 50526 899c9c4e4a4c
child 51002 496013a6eb38
equal deleted inserted replaced
50879:fc394c83e490 50880:b22ecedde1c7
   207     by simp
   207     by simp
   208 qed
   208 qed
   209 
   209 
   210 lemma isCont_vec_nth [simp]: "isCont f a \<Longrightarrow> isCont (\<lambda>x. f x $ i) a"
   210 lemma isCont_vec_nth [simp]: "isCont f a \<Longrightarrow> isCont (\<lambda>x. f x $ i) a"
   211   unfolding isCont_def by (rule tendsto_vec_nth)
   211   unfolding isCont_def by (rule tendsto_vec_nth)
   212 
       
   213 lemma eventually_Ball_finite: (* TODO: move *)
       
   214   assumes "finite A" and "\<forall>y\<in>A. eventually (\<lambda>x. P x y) net"
       
   215   shows "eventually (\<lambda>x. \<forall>y\<in>A. P x y) net"
       
   216 using assms by (induct set: finite, simp, simp add: eventually_conj)
       
   217 
       
   218 lemma eventually_all_finite: (* TODO: move *)
       
   219   fixes P :: "'a \<Rightarrow> 'b::finite \<Rightarrow> bool"
       
   220   assumes "\<And>y. eventually (\<lambda>x. P x y) net"
       
   221   shows "eventually (\<lambda>x. \<forall>y. P x y) net"
       
   222 using eventually_Ball_finite [of UNIV P] assms by simp
       
   223 
   212 
   224 lemma vec_tendstoI:
   213 lemma vec_tendstoI:
   225   assumes "\<And>i. ((\<lambda>x. f x $ i) ---> a $ i) net"
   214   assumes "\<And>i. ((\<lambda>x. f x $ i) ---> a $ i) net"
   226   shows "((\<lambda>x. f x) ---> a) net"
   215   shows "((\<lambda>x. f x) ---> a) net"
   227 proof (rule topological_tendstoI)
   216 proof (rule topological_tendstoI)