src/HOL/ex/Arithmetic_Series_Complex.thy
changeset 47223 4fc34c628474
parent 47222 1b7c909a6fad
child 47224 773fe2754b8c
--- a/src/HOL/ex/Arithmetic_Series_Complex.thy	Fri Mar 30 14:25:32 2012 +0200
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,17 +0,0 @@
-(*  Title:      HOL/ex/Arithmetic_Series_Complex.thy
-    Author:     Benjamin Porter, 2006
-*)
-
-
-header {* Arithmetic Series for Reals *}
-
-theory Arithmetic_Series_Complex
-imports "../RealDef"
-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))"
-  by (fact arith_series_general) (* FIXME: duplicate *)
-
-end