src/HOL/Complex/ex/ASeries_Complex.thy
changeset 19358 9cd12369e753
parent 19357 dade85a75c9f
child 19359 5d523a1b6ddc
--- a/src/HOL/Complex/ex/ASeries_Complex.thy	Fri Apr 07 11:17:44 2006 +0200
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,24 +0,0 @@
-(*  Title:      HOL/Library/ASeries.thy
-    ID:         $Id$
-    Author:     Benjamin Porter, 2006
-*)
-
-
-header {* Arithmetic Series for Reals *}
-
-theory ASeries_Complex
-imports Complex_Main ASeries
-begin
-
-lemma arith_series_real:
-  "(2::real) * (\<Sum>i\<in>{..<n}. a + of_nat i * d) =
-  of_nat n * (a + (a + of_nat(n - 1)*d))"
-proof -
-  have
-    "((1::real) + 1) * (\<Sum>i\<in>{..<n}. a + of_nat(i)*d) =
-    of_nat(n) * (a + (a + of_nat(n - 1)*d))"
-    by (rule arith_series_general)
-  thus ?thesis by simp
-qed
-
-end