src/Pure/Isar/specification.ML
changeset 46776 8575cc482dfb
parent 46728 85f8e3932712
child 46989 88b0a8052c75
--- a/src/Pure/Isar/specification.ML	Sat Mar 03 21:43:59 2012 +0100
+++ b/src/Pure/Isar/specification.ML	Sat Mar 03 21:52:15 2012 +0100
@@ -415,7 +415,7 @@
     |> (case facts of NONE => I | SOME ths => Proof.refine_insert ths)
     |> tap (fn state => not schematic andalso Proof.schematic_goal state andalso
         error "Illegal schematic goal statement")
-    |> Library.apply (map (fn (f, _) => f int) (rev (Theorem_Hook.get (Context.Proof goal_ctxt))))
+    |> fold_rev (fn (f, _) => f int) (Theorem_Hook.get (Context.Proof goal_ctxt))
   end;
 
 in