src/HOL/Codegenerator_Test/Generate.thy
changeset 37819 000049335247
parent 37745 6315b6426200
child 37824 365e37fe93f3
--- a/src/HOL/Codegenerator_Test/Generate.thy	Wed Jul 14 14:16:12 2010 +0200
+++ b/src/HOL/Codegenerator_Test/Generate.thy	Wed Jul 14 14:20:47 2010 +0200
@@ -15,15 +15,15 @@
 *}
 
 export_code "*" in SML module_name Code_Test file -
-ML {* Cache_IO.with_tmp_dir "Code_Test" (Code_ML.check_SML @{theory}) *}
+ML {* Code_ML.check_SML @{theory} *}
 
 export_code "*" in OCaml module_name Code_Test file -
-ML {* Cache_IO.with_tmp_dir "Code_Test" (Code_ML.check_OCaml @{theory}) *}
+ML {* Code_ML.check_OCaml @{theory} *}
 
 export_code "*" in Haskell module_name Code_Test file -
-ML {* Cache_IO.with_tmp_dir "Code_Test" (Code_Haskell.check @{theory}) *}
+ML {* Code_Haskell.check @{theory} *}
 
 export_code "*" in Scala module_name Code_Test file -
-ML {* Cache_IO.with_tmp_dir "Code_Test" (Code_Scala.check @{theory}) *}
+ML {* Code_Scala.check @{theory} *}
 
 end