src/ZF/ex/NatSum.thy
changeset 35762 af3ff2ba4c54
parent 16417 9bc16273c2d4
child 41777 1f7cbe39d425
--- a/src/ZF/ex/NatSum.thy	Sat Mar 13 16:37:15 2010 +0100
+++ b/src/ZF/ex/NatSum.thy	Sat Mar 13 16:44:12 2010 +0100
@@ -1,5 +1,4 @@
 (*  Title:      ZF/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.