author | haftmann |
Mon, 05 Jan 2009 15:37:49 +0100 | |
changeset 29359 | f831192b9366 |
parent 29295 | 93b819a44146 |
child 29514 | fc20414d4aa8 |
permissions | -rw-r--r-- |
28213 | 1 |
theory Setup |
28419 | 2 |
imports Complex_Main |
28440 | 3 |
uses "../../../antiquote_setup.ML" "../../../more_antiquote.ML" |
28213 | 4 |
begin |
5 |
||
28447 | 6 |
ML {* no_document use_thys |
28593 | 7 |
["Efficient_Nat", "Code_Char_chr", "Product_ord", "Imperative_HOL", |
29295 | 8 |
"~~/src/HOL/ex/ReflectedFerrack"] *} |
28419 | 9 |
|
28213 | 10 |
ML_val {* Code_Target.code_width := 74 *} |
11 |
||
12 |
end |