src/HOL/Code_Evaluation.thy
changeset 39401 887f4218a39a
parent 39387 6608c4838ff9
child 39403 aad9f3cfa1d9
equal deleted inserted replaced
39399:267235a14938 39401:887f4218a39a
   313 );
   313 );
   314 val put_term = Evaluation.put;
   314 val put_term = Evaluation.put;
   315 
   315 
   316 fun tracing s x = (Output.tracing s; x);
   316 fun tracing s x = (Output.tracing s; x);
   317 
   317 
   318 fun eval_term thy t = Code_Eval.eval NONE (Evaluation.get, put_term, "Code_Evaluation.put_term")
   318 fun eval_term thy t = Code_Runtime.eval NONE (Evaluation.get, put_term, "Code_Evaluation.put_term")
   319   I thy (HOLogic.mk_term_of (fastype_of t) t) [];
   319   I thy (HOLogic.mk_term_of (fastype_of t) t) [];
   320 
   320 
   321 end
   321 end
   322 *}
   322 *}
   323 
   323