src/HOL/SEQ.thy
changeset 31588 2651f172c38b
parent 31488 5691ccb8d6b5
child 32064 53ca12ff305d
--- a/src/HOL/SEQ.thy	Fri Jun 12 12:00:30 2009 -0700
+++ b/src/HOL/SEQ.thy	Fri Jun 12 15:46:21 2009 -0700
@@ -348,23 +348,7 @@
   fixes L :: "'a \<Rightarrow> 'b::real_normed_vector"
   assumes n: "\<And>n. n \<in> S \<Longrightarrow> X n ----> L n"
   shows "(\<lambda>m. \<Sum>n\<in>S. X n m) ----> (\<Sum>n\<in>S. L n)"
-proof (cases "finite S")
-  case True
-  thus ?thesis using n
-  proof (induct)
-    case empty
-    show ?case
-      by (simp add: LIMSEQ_const)
-  next
-    case insert
-    thus ?case
-      by (simp add: LIMSEQ_add)
-  qed
-next
-  case False
-  thus ?thesis
-    by (simp add: LIMSEQ_const)
-qed
+using n unfolding LIMSEQ_conv_tendsto by (rule tendsto_setsum)
 
 lemma LIMSEQ_setprod:
   fixes L :: "'a \<Rightarrow> 'b::{real_normed_algebra,comm_ring_1}"