src/HOL/Import/HOL4Setup.thy
changeset 17801 30cbd2685e73
parent 17322 781abf7011e6
child 19064 bf19cc5a7899
--- a/src/HOL/Import/HOL4Setup.thy	Sat Oct 08 22:39:38 2005 +0200
+++ b/src/HOL/Import/HOL4Setup.thy	Sat Oct 08 22:39:39 2005 +0200
@@ -4,7 +4,8 @@
 *)
 
 theory HOL4Setup imports MakeEqual
-  uses ("proof_kernel.ML") ("replay.ML") ("hol4rews.ML") ("import_package.ML") begin
+  uses "susp.ML" "lazy_seq.ML" "lazy_scan.ML"
+    ("proof_kernel.ML") ("replay.ML") ("hol4rews.ML") ("import_package.ML") begin
 
 section {* General Setup *}