src/HOL/Integ/NatSimprocs.thy
changeset 9436 62bb04ab4b01
parent 8858 b739f0ecc1fa
child 10536 8f34ecae1446
--- a/src/HOL/Integ/NatSimprocs.thy	Tue Jul 25 00:03:39 2000 +0200
+++ b/src/HOL/Integ/NatSimprocs.thy	Tue Jul 25 00:06:46 2000 +0200
@@ -1,2 +1,7 @@
-theory NatSimprocs = NatBin:
+
+theory NatSimprocs = NatBin
+files "nat_simprocs.ML":
+
+setup nat_simprocs_setup
+
 end