src/HOL/HOL.thy
changeset 59507 b468e0f8da2a
parent 59504 8c6747dba731
parent 59499 14095f771781
child 59582 0fbed69ff081
--- a/src/HOL/HOL.thy	Tue Feb 10 17:37:06 2015 +0000
+++ b/src/HOL/HOL.thy	Wed Feb 11 12:01:56 2015 +0000
@@ -846,8 +846,9 @@
   shows R
 apply (rule ex1E [OF major])
 apply (rule prem)
-apply (tactic {* ares_tac @{thms allI} 1 *})+
-apply (tactic {* eresolve_tac [Classical.dup_elim NONE @{thm allE}] 1 *})
+apply assumption
+apply (rule allI)+
+apply (tactic {* eresolve_tac @{context} [Classical.dup_elim NONE @{thm allE}] 1 *})
 apply iprover
 done
 
@@ -1796,7 +1797,7 @@
 proof
   assume "PROP ?ofclass"
   show "PROP ?equal"
-    by (tactic {* ALLGOALS (resolve_tac [Thm.unconstrainT @{thm eq_equal}]) *})
+    by (tactic {* ALLGOALS (resolve_tac @{context} [Thm.unconstrainT @{thm eq_equal}]) *})
       (fact `PROP ?ofclass`)
 next
   assume "PROP ?equal"
@@ -1897,7 +1898,7 @@
       let val conv = Code_Runtime.dynamic_holds_conv ctxt
       in
         CONVERSION (Conv.params_conv ~1 (K (Conv.concl_conv ~1 conv)) ctxt) THEN'
-        resolve_tac [TrueI]
+        resolve_tac ctxt [TrueI]
       end
   in
     Scan.succeed (SIMPLE_METHOD' o eval_tac)
@@ -1909,7 +1910,7 @@
     SIMPLE_METHOD'
       (CHANGED_PROP o
         (CONVERSION (Nbe.dynamic_conv ctxt)
-          THEN_ALL_NEW (TRY o resolve_tac [TrueI]))))
+          THEN_ALL_NEW (TRY o resolve_tac ctxt [TrueI]))))
 *} "solve goal by normalization"
 
 
@@ -1949,7 +1950,7 @@
     val filter_right = filter (not o wrong_prem o HOLogic.dest_Trueprop o hd o Thm.prems_of);
   in
     fun smp i = funpow i (fn m => filter_right ([spec] RL m)) ([mp]);
-    fun smp_tac ctxt j = EVERY'[dresolve_tac (smp j), assume_tac ctxt];
+    fun smp_tac ctxt j = EVERY' [dresolve_tac ctxt (smp j), assume_tac ctxt];
   end;
 
   local