src/Pure/Isar/expression.ML
changeset 58956 a816aa3ff391
parent 57926 59b2572e8e93
child 59296 002d817b4c37
--- a/src/Pure/Isar/expression.ML	Sun Nov 09 11:05:20 2014 +0100
+++ b/src/Pure/Isar/expression.ML	Sun Nov 09 14:08:00 2014 +0100
@@ -683,8 +683,9 @@
     val intro = Goal.prove_global defs_thy [] norm_ts statement
       (fn {context = ctxt, ...} =>
         rewrite_goals_tac ctxt [pred_def] THEN
-        compose_tac (false, body_eq RS Drule.equal_elim_rule1, 1) 1 THEN
-        compose_tac (false, Conjunction.intr_balanced (map (Thm.assume o cert) norm_ts), 0) 1);
+        compose_tac defs_ctxt (false, body_eq RS Drule.equal_elim_rule1, 1) 1 THEN
+        compose_tac defs_ctxt
+          (false, Conjunction.intr_balanced (map (Thm.assume o cert) norm_ts), 0) 1);
 
     val conjuncts =
       (Drule.equal_elim_rule2 OF
@@ -695,7 +696,7 @@
       |> Assumption.add_assumes (maps (#hyps o Thm.crep_thm) (defs @ conjuncts));
     val axioms = ts ~~ conjuncts |> map (fn (t, ax) =>
       Element.prove_witness axioms_ctxt t
-       (rewrite_goals_tac axioms_ctxt defs THEN compose_tac (false, ax, 0) 1));
+       (rewrite_goals_tac axioms_ctxt defs THEN compose_tac axioms_ctxt (false, ax, 0) 1));
   in ((statement, intro, axioms), defs_thy) end;
 
 in