author | kleing |
Wed, 11 Feb 2009 16:03:10 +1100 | |
changeset 29858 | c8cee17d7e50 |
parent 29794 | 32d00a2a6f28 |
child 30119 | 391e12ff816c |
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 |
29514 | 7 |
["Efficient_Nat", "Code_Char_chr", "Product_ord", "~~/src/HOL/Imperative_HOL/Imperative_HOL", |
29794 | 8 |
"~~/src/HOL/Reflection/Ferrack"] *} |
28419 | 9 |
|
28213 | 10 |
ML_val {* Code_Target.code_width := 74 *} |
11 |
||
12 |
end |