src/HOL/Library/Code_Char.thy
changeset 32657 5f13912245ff
parent 31053 b7e1c065b6e4
child 33226 a5eba0447559
     1.1 --- a/src/HOL/Library/Code_Char.thy	Wed Sep 23 13:42:53 2009 +0200
     1.2 +++ b/src/HOL/Library/Code_Char.thy	Wed Sep 23 14:00:12 2009 +0200
     1.3 @@ -5,7 +5,7 @@
     1.4  header {* Code generation of pretty characters (and strings) *}
     1.5  
     1.6  theory Code_Char
     1.7 -imports List Code_Eval Main
     1.8 +imports List Code_Evaluation Main
     1.9  begin
    1.10  
    1.11  code_type char
    1.12 @@ -32,7 +32,7 @@
    1.13    (OCaml "!((_ : char) = _)")
    1.14    (Haskell infixl 4 "==")
    1.15  
    1.16 -code_const "Code_Eval.term_of \<Colon> char \<Rightarrow> term"
    1.17 +code_const "Code_Evaluation.term_of \<Colon> char \<Rightarrow> term"
    1.18    (Eval "HOLogic.mk'_char/ (IntInf.fromInt/ (Char.ord/ _))")
    1.19  
    1.20  end