src/Doc/Codegen/Setup.thy
changeset 59378 065f349852e6
parent 59377 056945909f60
child 61143 5f898411ce87
--- a/src/Doc/Codegen/Setup.thy	Thu Jan 15 13:39:41 2015 +0100
+++ b/src/Doc/Codegen/Setup.thy	Thu Jan 15 13:39:41 2015 +0100
@@ -1,16 +1,13 @@
 theory Setup
 imports
   Complex_Main
+  "~~/src/Tools/Permanent_Interpretation"
   "~~/src/HOL/Library/Dlist"
   "~~/src/HOL/Library/RBT"
   "~~/src/HOL/Library/Mapping"
   "~~/src/HOL/Library/IArray"
 begin
 
-ML \<open>
-  Isabelle_System.mkdirs (File.tmp_path (Path.basic "examples"))
-\<close>
-
 ML_file "../antiquote_setup.ML"
 ML_file "../more_antiquote.ML"