src/FOL/ex/Natural_Numbers.thy
changeset 31974 e81979a703a4
parent 26720 8d1925ad0dac
child 44605 4877c4e184e5
--- a/src/FOL/ex/Natural_Numbers.thy	Thu Jul 09 22:04:10 2009 +0200
+++ b/src/FOL/ex/Natural_Numbers.thy	Thu Jul 09 22:09:58 2009 +0200
@@ -1,11 +1,12 @@
 (*  Title:      FOL/ex/Natural_Numbers.thy
-    ID:         $Id$
     Author:     Markus Wenzel, TU Munich
 *)
 
 header {* Natural numbers *}
 
-theory Natural_Numbers imports FOL begin
+theory Natural_Numbers
+imports FOL
+begin
 
 text {*
   Theory of the natural numbers: Peano's axioms, primitive recursion.