| author | wenzelm | 
| Tue, 03 Aug 2010 18:10:18 +0200 | |
| changeset 38138 | dc65ed8bbb43 | 
| parent 34071 | 93bfbb557e2e | 
| child 38460 | 628fee3eb449 | 
| permissions | -rw-r--r-- | 
| 28213 | 1 | theory Setup | 
| 28419 | 2 | imports Complex_Main | 
| 30227 | 3 | uses | 
| 4 | "../../antiquote_setup.ML" | |
| 5 | "../../more_antiquote.ML" | |
| 28213 | 6 | begin | 
| 7 | ||
| 28447 | 8 | ML {* no_document use_thys
 | 
| 29514 | 9 | ["Efficient_Nat", "Code_Char_chr", "Product_ord", "~~/src/HOL/Imperative_HOL/Imperative_HOL", | 
| 30119 
391e12ff816c
fixed import of ~~/src/HOL/Decision_Procs/Ferrack;
 wenzelm parents: 
29794diff
changeset | 10 | "~~/src/HOL/Decision_Procs/Ferrack"] *} | 
| 28419 | 11 | |
| 34071 | 12 | setup {* Code_Target.set_default_code_width 74 *}
 | 
| 13 | ||
| 32833 | 14 | ML_command {* Unsynchronized.reset unique_names *}
 | 
| 28213 | 15 | |
| 16 | end |