| author | haftmann | 
| Tue, 26 May 2009 12:31:01 +0200 | |
| changeset 31254 | 03a35fbc9dc6 | 
| parent 30227 | 853abb4853cc | 
| child 32833 | f3716d1a2e48 | 
| 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 | |
| 30227 | 12 | ML_command {* Code_Target.code_width := 74 *}
 | 
| 13 | ML_command {* reset unique_names *}
 | |
| 28213 | 14 | |
| 15 | end |