src/HOL/Tools/Predicate_Compile/predicate_compile_fun.ML
changeset 35021 c839a4c670c6
parent 34954 b206c70ea6f0
child 35324 c9f428269b38
--- a/src/HOL/Tools/Predicate_Compile/predicate_compile_fun.ML	Sun Feb 07 19:31:55 2010 +0100
+++ b/src/HOL/Tools/Predicate_Compile/predicate_compile_fun.ML	Sun Feb 07 19:33:34 2010 +0100
@@ -391,7 +391,7 @@
         |> map (fn (concl'::conclprems, _) =>
           Logic.list_implies ((flat prems') @ conclprems, concl')))
   in
-    map (Drule.standard o (Skip_Proof.make_thm thy)) intro_ts'
+    map (Drule.export_without_context o Skip_Proof.make_thm thy) intro_ts'
   end
 
 end;