src/HOL/Multivariate_Analysis/Finite_Cartesian_Product.thy
changeset 61810 3c5040d5694a
parent 61169 4de9ff3ea29a
child 61969 e01015e49041
equal deleted inserted replaced
61809:81d34cf268d8 61810:3c5040d5694a
   222   have "\<And>i. eventually (\<lambda>x. f x $ i \<in> A i) net"
   222   have "\<And>i. eventually (\<lambda>x. f x $ i \<in> A i) net"
   223     using assms A by (rule topological_tendstoD)
   223     using assms A by (rule topological_tendstoD)
   224   hence "eventually (\<lambda>x. \<forall>i. f x $ i \<in> A i) net"
   224   hence "eventually (\<lambda>x. \<forall>i. f x $ i \<in> A i) net"
   225     by (rule eventually_all_finite)
   225     by (rule eventually_all_finite)
   226   thus "eventually (\<lambda>x. f x \<in> S) net"
   226   thus "eventually (\<lambda>x. f x \<in> S) net"
   227     by (rule eventually_elim1, simp add: S)
   227     by (rule eventually_mono, simp add: S)
   228 qed
   228 qed
   229 
   229 
   230 lemma tendsto_vec_lambda [tendsto_intros]:
   230 lemma tendsto_vec_lambda [tendsto_intros]:
   231   assumes "\<And>i. ((\<lambda>x. f x i) ---> a i) net"
   231   assumes "\<And>i. ((\<lambda>x. f x i) ---> a i) net"
   232   shows "((\<lambda>x. \<chi> i. f x i) ---> (\<chi> i. a i)) net"
   232   shows "((\<lambda>x. \<chi> i. f x i) ---> (\<chi> i. a i)) net"