src/FOL/ex/Natural_Numbers.thy
changeset 16417 9bc16273c2d4
parent 14981 e73f8140af78
child 25989 3267d0694d93
--- a/src/FOL/ex/Natural_Numbers.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/FOL/ex/Natural_Numbers.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -5,7 +5,7 @@
 
 header {* Natural numbers *}
 
-theory Natural_Numbers = FOL:
+theory Natural_Numbers imports FOL begin
 
 text {*
   Theory of the natural numbers: Peano's axioms, primitive recursion.