src/HOL/Import/Generate-HOL/GenHOL4Vec.thy
changeset 46780 ab4f3f765f91
parent 41589 bbd861837ebc
--- a/src/HOL/Import/Generate-HOL/GenHOL4Vec.thy	Sat Mar 03 14:04:49 2012 +0100
+++ b/src/HOL/Import/Generate-HOL/GenHOL4Vec.thy	Sat Mar 03 21:00:04 2012 +0100
@@ -10,29 +10,29 @@
 
 append_dump "theory HOL4Vec imports HOL4Base begin";
 
-import_theory res_quan;
+import_theory "~~/src/HOL/Import/HOL" res_quan;
 end_import;
 
-import_theory word_base;
+import_theory "~~/src/HOL/Import/HOL" word_base;
 
 const_renames
   BIT > bit;
 
 end_import;
 
-import_theory word_num;
+import_theory "~~/src/HOL/Import/HOL" word_num;
 end_import;
 
-import_theory word_bitop;
+import_theory "~~/src/HOL/Import/HOL" word_bitop;
 end_import;
 
-import_theory bword_num;
+import_theory "~~/src/HOL/Import/HOL" bword_num;
 end_import;
 
-import_theory bword_arith;
+import_theory "~~/src/HOL/Import/HOL" bword_arith;
 end_import;
 
-import_theory bword_bitop;
+import_theory "~~/src/HOL/Import/HOL" bword_bitop;
 end_import;
 
 append_dump "end";