src/HOL/MicroJava/J/JTypeSafe.thy
changeset 60754 02924903a6fd
parent 59826 442b09c0f898
child 61361 8b5f00202e1a
--- a/src/HOL/MicroJava/J/JTypeSafe.thy	Sat Jul 18 20:53:05 2015 +0200
+++ b/src/HOL/MicroJava/J/JTypeSafe.thy	Sat Jul 18 20:54:56 2015 +0200
@@ -178,8 +178,9 @@
 
 ML{*
 fun forward_hyp_tac ctxt =
-  ALLGOALS (TRY o (EVERY' [dtac spec, mp_tac ctxt,
-    (mp_tac ctxt ORELSE' (dtac spec THEN' mp_tac ctxt)), REPEAT o (etac conjE)]))
+  ALLGOALS (TRY o (EVERY' [dresolve_tac ctxt [spec], mp_tac ctxt,
+    (mp_tac ctxt ORELSE' (dresolve_tac ctxt [spec] THEN' mp_tac ctxt)),
+    REPEAT o (eresolve_tac ctxt [conjE])]))
 *}
 
 
@@ -202,7 +203,7 @@
 apply( tactic "ALLGOALS (REPEAT o resolve_tac @{context} [impI, allI])")
 apply( tactic {* ALLGOALS (eresolve_tac @{context} [@{thm ty_expr.cases}, @{thm ty_exprs.cases}, @{thm wt_stmt.cases}]
   THEN_ALL_NEW (full_simp_tac (put_simpset (simpset_of @{theory_context Conform}) @{context}))) *})
-apply(tactic "ALLGOALS (EVERY' [REPEAT o (etac conjE), REPEAT o hyp_subst_tac @{context}])")
+apply(tactic "ALLGOALS (EVERY' [REPEAT o (eresolve_tac @{context} [conjE]), REPEAT o hyp_subst_tac @{context}])")
 
 -- "Level 7"
 -- "15 NewC"
@@ -241,7 +242,7 @@
 
 -- "for FAss"
 apply( tactic {* EVERY'[eresolve_tac @{context} [@{thm ty_expr.cases}, @{thm ty_exprs.cases}, @{thm wt_stmt.cases}] 
-       THEN_ALL_NEW (full_simp_tac @{context}), REPEAT o (etac conjE), hyp_subst_tac @{context}] 3*})
+       THEN_ALL_NEW (full_simp_tac @{context}), REPEAT o (eresolve_tac @{context} [conjE]), hyp_subst_tac @{context}] 3*})
 
 -- "for if"
 apply( tactic {* (Induct_Tacs.case_tac @{context} "the_Bool v" [] NONE THEN_ALL_NEW