src/ZF/ex/NatSum.thy
changeset 9647 e9623f47275b
child 12867 5c900a821a7c
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/ZF/ex/NatSum.thy	Fri Aug 18 12:31:20 2000 +0200
@@ -0,0 +1,18 @@
+(*  Title:      HOL/ex/Natsum.thy
+    ID:         $Id$
+    Author:     Tobias Nipkow & Lawrence C Paulson
+
+A summation operator. sum(f,n+1) is the sum of all f(i), i=0...n.
+
+Note: n is a natural number but the sum is an integer,
+                            and f maps integers to integers
+*)
+
+NatSum = Main +
+
+consts sum     :: [i=>i, i] => i
+primrec 
+  "sum (f,0) = #0"
+  "sum (f, succ(n)) = f($#n) $+ sum(f,n)"
+
+end
\ No newline at end of file