doc-src/Codegen/Thy/Setup.thy
changeset 46517 9d2e682a68eb
parent 43564 9864182c6bad
child 48891 c0eafbd55de3
--- a/doc-src/Codegen/Thy/Setup.thy	Sat Feb 18 20:06:59 2012 +0100
+++ b/doc-src/Codegen/Thy/Setup.thy	Sat Feb 18 20:07:26 2012 +0100
@@ -1,7 +1,9 @@
 theory Setup
 imports
   Complex_Main
-  More_List RBT Dlist List_Cset Mapping
+  "~~/src/HOL/Library/Dlist"
+  "~~/src/HOL/Library/RBT"
+  "~~/src/HOL/Library/Mapping"
 uses
   "../../antiquote_setup.ML"
   "../../more_antiquote.ML"
@@ -27,3 +29,4 @@
 declare [[names_unique = false]]
 
 end
+