remove content-free theory ex/Arithmetic_Series_Complex.thy
authorhuffman
Fri, 30 Mar 2012 14:27:29 +0200
changeset 47223 4fc34c628474
parent 47222 1b7c909a6fad
child 47224 773fe2754b8c
remove content-free theory ex/Arithmetic_Series_Complex.thy
src/HOL/IsaMakefile
src/HOL/ex/Arithmetic_Series_Complex.thy
src/HOL/ex/ROOT.ML
--- a/src/HOL/IsaMakefile	Fri Mar 30 14:25:32 2012 +0200
+++ b/src/HOL/IsaMakefile	Fri Mar 30 14:27:29 2012 +0200
@@ -1128,7 +1128,7 @@
   Library/Code_Integer.thy Library/Code_Nat.thy				\
   Library/Code_Natural.thy Library/Efficient_Nat.thy			\
   Number_Theory/Primes.thy ex/Abstract_NAT.thy ex/Antiquote.thy		\
-  ex/Arith_Examples.thy ex/Arithmetic_Series_Complex.thy ex/BT.thy	\
+  ex/Arith_Examples.thy ex/BT.thy					\
   ex/BinEx.thy ex/Binary.thy ex/Birthday_Paradox.thy ex/CTL.thy		\
   ex/Case_Product.thy ex/Chinese.thy ex/Classical.thy			\
   ex/Code_Nat_examples.thy						\
--- 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
--- a/src/HOL/ex/ROOT.ML	Fri Mar 30 14:25:32 2012 +0200
+++ b/src/HOL/ex/ROOT.ML	Fri Mar 30 14:27:29 2012 +0200
@@ -57,7 +57,6 @@
   "Sqrt",
   "Sqrt_Script",
   "Transfer_Ex",
-  "Arithmetic_Series_Complex",
   "HarmonicSeries",
   "Refute_Examples",
   "Landau",