src/FOL/ex/NatClass.thy
changeset 17274 746bb4c56800
parent 17245 1c519a3cca59
child 19819 14de4d05d275
--- a/src/FOL/ex/NatClass.thy	Tue Sep 06 16:29:39 2005 +0200
+++ b/src/FOL/ex/NatClass.thy	Tue Sep 06 16:59:48 2005 +0200
@@ -34,6 +34,6 @@
   "m + n == rec(m, n, %x y. Suc(y))"
 
 ML {* use_legacy_bindings (the_context ()) *}
-ML {* open nat *}
+ML {* open nat_class *}
 
 end