doc-src/Codegen/Thy/Setup.thy
changeset 30227 853abb4853cc
parent 30226 2f4684e2ea95
child 32833 f3716d1a2e48
--- a/doc-src/Codegen/Thy/Setup.thy	Tue Mar 03 11:00:51 2009 +0100
+++ b/doc-src/Codegen/Thy/Setup.thy	Tue Mar 03 13:20:53 2009 +0100
@@ -1,12 +1,15 @@
 theory Setup
 imports Complex_Main
-uses "../../../antiquote_setup.ML" "../../../more_antiquote.ML"
+uses
+  "../../antiquote_setup.ML"
+  "../../more_antiquote.ML"
 begin
 
 ML {* no_document use_thys
   ["Efficient_Nat", "Code_Char_chr", "Product_ord", "~~/src/HOL/Imperative_HOL/Imperative_HOL",
    "~~/src/HOL/Decision_Procs/Ferrack"] *}
 
-ML_val {* Code_Target.code_width := 74 *}
+ML_command {* Code_Target.code_width := 74 *}
+ML_command {* reset unique_names *}
 
 end