src/HOL/Code_Eval.thy
changeset 30970 3fe2e418a071
parent 30947 dd551284a300
child 31031 cbec39ebf8f2
--- a/src/HOL/Code_Eval.thy	Fri Apr 24 08:24:52 2009 +0200
+++ b/src/HOL/Code_Eval.thy	Fri Apr 24 08:24:54 2009 +0200
@@ -161,6 +161,7 @@
 signature EVAL =
 sig
   val mk_term: ((string * typ) -> term) -> (typ -> term) -> term -> term
+  val mk_term_of: typ -> term -> term
   val eval_ref: (unit -> term) option ref
   val eval_term: theory -> term -> term
 end;
@@ -175,7 +176,7 @@
 fun eval_term thy t =
   t 
   |> Eval.mk_term_of (fastype_of t)
-  |> (fn t => Code_ML.eval_term NONE ("Eval.eval_ref", eval_ref) thy t []);
+  |> (fn t => Code_ML.eval NONE ("Eval.eval_ref", eval_ref) I thy t []);
 
 end;
 *}