doc-src/IsarAdvanced/Codegen/Thy/Setup.thy
changeset 30226 2f4684e2ea95
parent 30202 2775062fd3a9
child 30227 853abb4853cc
--- a/doc-src/IsarAdvanced/Codegen/Thy/Setup.thy	Mon Mar 02 16:58:39 2009 +0100
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,12 +0,0 @@
-theory Setup
-imports Complex_Main
-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 *}
-
-end