use \<Sum> from main HOL;
authorwenzelm
Thu, 14 Dec 2000 19:37:09 +0100
changeset 10672 3b1c2d74a01b
parent 10671 ac6b3b671198
child 10673 337c00fd385b
use \<Sum> from main HOL;
src/HOL/Isar_examples/Summation.thy
--- a/src/HOL/Isar_examples/Summation.thy	Thu Dec 14 19:36:48 2000 +0100
+++ b/src/HOL/Isar_examples/Summation.thy	Thu Dec 14 19:37:09 2000 +0100
@@ -22,31 +22,6 @@
 *}
 
 
-subsection {* A summation operator *}
-
-text {*
-  The binder operator $\idt{sum} :: (\idt{nat} \To \idt{nat}) \To
- \idt{nat} \To \idt{nat}$ formalizes summation of natural numbers
- indexed from $0$ up to $k$ (excluding the bound):
- \[
- \sum\limits_{i < k} f(i) = \idt{sum} \ap (\lam i f \ap i) \ap k
- \]
-*}
-
-consts
-  sum :: "(nat => nat) => nat => nat"
-
-primrec
-  "sum f 0 = 0"
-  "sum f (Suc n) = f n + sum f n"
-
-syntax
-  "_SUM" :: "idt => nat => nat => nat"
-    ("SUM _ < _. _" [0, 0, 10] 10)
-translations
-  "SUM i < k. b" == "sum (\<lambda>i. b) k"
-
-
 subsection {* Summation laws *}
 
 text {*
@@ -56,7 +31,7 @@
 *}
 
 theorem sum_of_naturals:
-  "2 * (SUM i < n + 1. i) = n * (n + 1)"
+  "2 * (\<Sum>i < n + 1. i) = n * (n + 1)"
   (is "?P n" is "?S n = _")
 proof (induct n)
   show "?P 0" by simp
@@ -111,7 +86,7 @@
 *}
 
 theorem sum_of_odds:
-  "(SUM i < n. 2 * i + 1) = n^2"
+  "(\<Sum>i < n. 2 * i + 1) = n^2"
   (is "?P n" is "?S n = _")
 proof (induct n)
   show "?P 0" by simp
@@ -131,7 +106,7 @@
 lemmas distrib = add_mult_distrib add_mult_distrib2
 
 theorem sum_of_squares:
-  "#6 * (SUM i < n + 1. i^2) = n * (n + 1) * (2 * n + 1)"
+  "#6 * (\<Sum>i < n + 1. i^2) = n * (n + 1) * (2 * n + 1)"
   (is "?P n" is "?S n = _")
 proof (induct n)
   show "?P 0" by simp
@@ -144,7 +119,7 @@
 qed
 
 theorem sum_of_cubes:
-  "#4 * (SUM i < n + 1. i^#3) = (n * (n + 1))^2"
+  "#4 * (\<Sum>i < n + 1. i^#3) = (n * (n + 1))^2"
   (is "?P n" is "?S n = _")
 proof (induct n)
   show "?P 0" by (simp add: power_eq_if)