src/HOL/Library/Code_Integer.thy
changeset 31192 a324d214009c
parent 30663 0b6aff7451b2
child 31203 5c8fb4fd67e0
     1.1 --- a/src/HOL/Library/Code_Integer.thy	Mon May 18 15:45:32 2009 +0200
     1.2 +++ b/src/HOL/Library/Code_Integer.thy	Mon May 18 15:45:34 2009 +0200
     1.3 @@ -5,7 +5,7 @@
     1.4  header {* Pretty integer literals for code generation *}
     1.5  
     1.6  theory Code_Integer
     1.7 -imports Main
     1.8 +imports Main Code_Index
     1.9  begin
    1.10  
    1.11  text {*
    1.12 @@ -91,15 +91,17 @@
    1.13    (OCaml "Big'_int.lt'_big'_int")
    1.14    (Haskell infix 4 "<")
    1.15  
    1.16 +code_const Code_Index.int_of
    1.17 +  (SML "IntInf.fromInt")
    1.18 +  (OCaml "Big'_int.big'_int'_of'_int")
    1.19 +  (Haskell "toEnum")
    1.20 +
    1.21  code_reserved SML IntInf
    1.22  code_reserved OCaml Big_int
    1.23  
    1.24  text {* Evaluation *}
    1.25  
    1.26 -lemma [code, code del]:
    1.27 -  "(Code_Eval.term_of \<Colon> int \<Rightarrow> term) = Code_Eval.term_of" ..
    1.28 -
    1.29  code_const "Code_Eval.term_of \<Colon> int \<Rightarrow> term"
    1.30 -  (SML "HOLogic.mk'_number/ HOLogic.intT")
    1.31 +  (Eval "HOLogic.mk'_number/ HOLogic.intT")
    1.32  
    1.33  end
    1.34 \ No newline at end of file