add bounded_linear lemmas
authorhuffman
Tue, 29 May 2007 17:37:04 +0200
changeset 23119 0082459a255b
parent 23118 ce3cf072ae14
child 23120 a34f204e9c88
add bounded_linear lemmas
src/HOL/Hyperreal/Series.thy
--- a/src/HOL/Hyperreal/Series.thy	Tue May 29 17:36:35 2007 +0200
+++ b/src/HOL/Hyperreal/Series.thy	Tue May 29 17:37:04 2007 +0200
@@ -164,6 +164,18 @@
   apply (rule sums_zero);
 done;
   
+lemma (in bounded_linear) sums:
+  "(\<lambda>n. X n) sums a \<Longrightarrow> (\<lambda>n. f (X n)) sums (f a)"
+unfolding sums_def by (drule LIMSEQ, simp only: setsum)
+
+lemma (in bounded_linear) summable:
+  "summable (\<lambda>n. X n) \<Longrightarrow> summable (\<lambda>n. f (X n))"
+unfolding summable_def by (auto intro: sums)
+
+lemma (in bounded_linear) suminf:
+  "summable (\<lambda>n. X n) \<Longrightarrow> f (\<Sum>n. X n) = (\<Sum>n. f (X n))"
+by (rule summable_sums [THEN sums, THEN sums_unique])
+
 lemma sums_mult:
   fixes c :: "'a::real_normed_algebra"
   shows "f sums a \<Longrightarrow> (\<lambda>n. c * f n) sums (c * a)"