| author | wenzelm |
| Thu, 23 Oct 2008 13:52:27 +0200 | |
| changeset 28671 | ed6681dd35d8 |
| parent 28593 | f087237af65d |
| child 29295 | 93b819a44146 |
| 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", |
8 |
"~~/src/HOL/Complex/ex/ReflectedFerrack"] *} |
|
| 28419 | 9 |
|
| 28213 | 10 |
ML_val {* Code_Target.code_width := 74 *}
|
11 |
||
12 |
end |