src/Pure/codegen.ML
changeset 32970 fbd2bb2489a8
parent 32966 5b21661fe618
child 33001 82382652e5e7
--- a/src/Pure/codegen.ML	Sat Oct 17 16:40:41 2009 +0200
+++ b/src/Pure/codegen.ML	Sat Oct 17 16:58:03 2009 +0200
@@ -280,8 +280,7 @@
   let
     val x = Free (Name.variant (OldTerm.add_term_names (t, [])) "x", fastype_of t);
     (* fake definition *)
-    val eq = setmp_CRITICAL quick_and_dirty true (SkipProof.make_thm thy)
-      (Logic.mk_equals (x, t));
+    val eq = Skip_Proof.make_thm thy (Logic.mk_equals (x, t));
     fun err () = error "preprocess_term: bad preprocessor"
   in case map prop_of (preprocess thy [eq]) of
       [Const ("==", _) $ x' $ t'] => if x = x' then t' else err ()