src/HOL/ex/Predicate_Compile.thy
changeset 31140 e5f8c1c420f3
parent 31129 d2cead76fca2
child 31217 c025f32afd4e
--- a/src/HOL/ex/Predicate_Compile.thy	Wed May 13 18:41:54 2009 +0200
+++ b/src/HOL/ex/Predicate_Compile.thy	Wed May 13 18:48:17 2009 +0200
@@ -22,9 +22,7 @@
 val pred_ref = ref (NONE : (unit -> term Predicate.pred) option);
 
 fun eval_pred thy t =
-  t 
-  |> Eval.mk_term_of (fastype_of t)
-  |> (fn t => Code_ML.eval NONE ("Predicate.pred_ref", pred_ref) @{code pred_map} thy t []);
+  Code_ML.eval NONE ("Predicate.pred_ref", pred_ref) @{code pred_map} thy (HOLogic.mk_term_of (fastype_of t) t) [];
 
 fun eval_pred_elems thy t T length =
   t |> eval_pred thy |> yieldn length |> fst |> HOLogic.mk_list T;