src/HOL/Library/Efficient_Nat.thy
changeset 28228 7ebe8dc06cbb
parent 27673 52056ddac194
child 28346 b8390cd56b8f
--- a/src/HOL/Library/Efficient_Nat.thy	Tue Sep 16 09:21:22 2008 +0200
+++ b/src/HOL/Library/Efficient_Nat.thy	Tue Sep 16 09:21:24 2008 +0200
@@ -6,7 +6,7 @@
 header {* Implementation of natural numbers by target-language integers *}
 
 theory Efficient_Nat
-imports Plain Code_Integer Code_Index
+imports Plain Code_Index Code_Integer
 begin
 
 text {*
@@ -424,6 +424,15 @@
   "op < \<Colon>  nat \<Rightarrow> nat \<Rightarrow> bool"  ("(_ </ _)")
 
 
+text {* Evaluation *}
+
+lemma [code func, code func del]:
+  "(Code_Eval.term_of \<Colon> nat \<Rightarrow> term) = Code_Eval.term_of" ..
+
+code_const "Code_Eval.term_of \<Colon> nat \<Rightarrow> term"
+  (SML "HOLogic.mk'_number/ HOLogic.natT")
+
+
 text {* Module names *}
 
 code_modulename SML