src/HOL/Library/Code_Integer.thy
changeset 28228 7ebe8dc06cbb
parent 27487 c8a6ce181805
child 28346 b8390cd56b8f
     1.1 --- a/src/HOL/Library/Code_Integer.thy	Tue Sep 16 09:21:22 2008 +0200
     1.2 +++ b/src/HOL/Library/Code_Integer.thy	Tue Sep 16 09:21:24 2008 +0200
     1.3 @@ -6,7 +6,7 @@
     1.4  header {* Pretty integer literals for code generation *}
     1.5  
     1.6  theory Code_Integer
     1.7 -imports Plain "~~/src/HOL/Presburger"
     1.8 +imports Plain "~~/src/HOL/Code_Eval" "~~/src/HOL/Presburger"
     1.9  begin
    1.10  
    1.11  text {*
    1.12 @@ -90,4 +90,12 @@
    1.13  code_reserved SML IntInf
    1.14  code_reserved OCaml Big_int
    1.15  
    1.16 +text {* Evaluation *}
    1.17 +
    1.18 +lemma [code func, code func del]:
    1.19 +  "(Code_Eval.term_of \<Colon> int \<Rightarrow> term) = Code_Eval.term_of" ..
    1.20 +
    1.21 +code_const "Code_Eval.term_of \<Colon> int \<Rightarrow> term"
    1.22 +  (SML "HOLogic.mk'_number/ HOLogic.intT")
    1.23 +
    1.24  end
    1.25 \ No newline at end of file