| 24195 |      1 | (*  Title:      HOL/ex/Codegenerator_Pretty.thy
 | 
|  |      2 |     ID:         $Id$
 | 
|  |      3 |     Author:     Florian Haftmann, TU Muenchen
 | 
|  |      4 | *)
 | 
|  |      5 | 
 | 
|  |      6 | header {* Simple examples for pretty numerals and such *}
 | 
|  |      7 | 
 | 
|  |      8 | theory Codegenerator_Pretty
 | 
| 25963 |      9 | imports ExecutableContent Code_Char Efficient_Nat
 | 
| 24195 |     10 | begin
 | 
|  |     11 | 
 | 
| 28562 |     12 | declare isnorm.simps [code del]
 | 
| 28228 |     13 | 
 | 
| 25963 |     14 | ML {* (*FIXME get rid of this*)
 | 
|  |     15 | nonfix union;
 | 
|  |     16 | nonfix inter;
 | 
|  |     17 | nonfix upto;
 | 
|  |     18 | *}
 | 
| 25933 |     19 | 
 | 
| 25963 |     20 | export_code * in SML module_name CodegenTest
 | 
|  |     21 |   in OCaml module_name CodegenTest file -
 | 
|  |     22 |   in Haskell file -
 | 
| 25616 |     23 | 
 | 
| 25963 |     24 | ML {*
 | 
|  |     25 | infix union;
 | 
|  |     26 | infix inter;
 | 
|  |     27 | infix 4 upto;
 | 
|  |     28 | *}
 | 
| 24195 |     29 | 
 | 
|  |     30 | end
 |