| author | wenzelm | 
| Sat, 03 Sep 2011 21:15:35 +0200 | |
| changeset 44676 | 7de87f1ae965 | 
| parent 42842 | 6ef538f6a8ab | 
| child 51143 | 0a2371e7ced3 | 
| permissions | -rw-r--r-- | 
| 24195 | 1 | |
| 31378 | 2 | (* Author: Florian Haftmann, TU Muenchen *) | 
| 3 | ||
| 4 | header {* Generating code using pretty literals and natural number literals  *}
 | |
| 24195 | 5 | |
| 37695 
71e84a203c19
introduced distinct session HOL-Codegenerator_Test
 haftmann parents: 
31378diff
changeset | 6 | theory Candidates_Pretty | 
| 42842 
6ef538f6a8ab
adding Code_Char_ord to code generation regression tests
 bulwahn parents: 
37695diff
changeset | 7 | imports Candidates Code_Char_ord Efficient_Nat | 
| 24195 | 8 | begin | 
| 9 | ||
| 10 | end |