src/HOL/Library/Eval.thy
changeset 24916 dc56dd1b3cda
parent 24867 e5b55d7be9bb
child 24920 2a45e400fdad
equal deleted inserted replaced
24915:fc90277c0dd7 24916:dc56dd1b3cda
   167 struct
   167 struct
   168 
   168 
   169 val eval_ref = ref (NONE : (unit -> term) option);
   169 val eval_ref = ref (NONE : (unit -> term) option);
   170 
   170 
   171 fun eval_invoke thy code ((_, ty), t) deps _ =
   171 fun eval_invoke thy code ((_, ty), t) deps _ =
   172   CodePackage.eval_invoke thy ("Eval.eval_ref", eval_ref) code (t, ty) [];
   172   CodeTarget.eval_invoke thy ("Eval.eval_ref", eval_ref) code (t, ty) [];
   173 
   173 
   174 fun eval_term thy =
   174 fun eval_term thy =
   175   TermOf.mk_term_of
   175   TermOf.mk_term_of
   176   #> CodePackage.eval_term thy (eval_invoke thy)
   176   #> CodePackage.eval_term thy (eval_invoke thy)
   177   #> Code.postprocess_term thy;
   177   #> Code.postprocess_term thy;