src/Pure/Isar/proof.ML
changeset 58950 d07464875dd4
parent 58892 20aa19ecf2cc
child 59150 71b416020f42
--- a/src/Pure/Isar/proof.ML	Sat Nov 08 17:39:01 2014 +0100
+++ b/src/Pure/Isar/proof.ML	Sat Nov 08 21:31:51 2014 +0100
@@ -471,7 +471,7 @@
     val th =
       (Goal.conclude (if length (flat propss) > 1 then Thm.norm_proof goal else goal)
         handle THM _ => lost_structure ())
-      |> Drule.flexflex_unique
+      |> Drule.flexflex_unique (SOME ctxt)
       |> Thm.check_shyps (Variable.sorts_of ctxt)
       |> Thm.check_hyps (Context.Proof ctxt);
 
@@ -480,8 +480,9 @@
       Conjunction.elim_balanced (length goal_propss) th
       |> map2 Conjunction.elim_balanced (map length goal_propss)
       handle THM _ => lost_structure ();
-    val _ = Unify.matches_list thy (flat goal_propss) (map Thm.prop_of (flat results)) orelse
-      error ("Proved a different theorem:\n" ^ Display.string_of_thm ctxt th);
+    val _ =
+      Unify.matches_list (Context.Proof ctxt) (flat goal_propss) (map Thm.prop_of (flat results))
+        orelse error ("Proved a different theorem:\n" ^ Display.string_of_thm ctxt th);
 
     fun recover_result ([] :: pss) thss = [] :: recover_result pss thss
       | recover_result (_ :: pss) (ths :: thss) = ths :: recover_result pss thss