theorem hooks: apply in declaration order;
authorwenzelm
Thu, 06 Sep 2007 12:30:11 +0200
changeset 24542 f13c59e40617
parent 24541 98c978a42a42
child 24543 e2332d1ff6c7
theorem hooks: apply in declaration order;
src/Pure/Isar/specification.ML
--- a/src/Pure/Isar/specification.ML	Thu Sep 06 11:53:17 2007 +0200
+++ b/src/Pure/Isar/specification.ML	Thu Sep 06 12:30:11 2007 +0200
@@ -289,8 +289,7 @@
     |> ProofContext.note_thmss_i Thm.assumptionK [((AutoBind.assmsN, []), [(prems, [])])]
     |> snd
     |> Proof.theorem_i before_qed after_qed' (map snd stmt)
-    |> Library.apply (map (fn (f, _) => f int)
-      (TheoremHook.get (Context.Proof goal_ctxt)))
+    |> Library.apply (map (fn (f, _) => f int) (rev (TheoremHook.get (Context.Proof goal_ctxt))))
     |> Proof.refine_insert facts
   end;