src/HOL/Bali/WellType.thy
changeset 59498 50b60f501b05
parent 58887 38db8ddc0f57
child 59763 56d2c357e6b5
--- a/src/HOL/Bali/WellType.thy	Tue Feb 10 14:29:36 2015 +0100
+++ b/src/HOL/Bali/WellType.thy	Tue Feb 10 14:48:26 2015 +0100
@@ -665,7 +665,7 @@
     thin_tac @{context} "?E,dt\<Turnstile>e2\<Colon>-?T2"] i
   else thin_tac @{context} "All ?P" i) *})
 (*apply (safe del: disjE elim!: wt_elim_cases)*)
-apply (tactic {*ALLGOALS (eresolve_tac @{thms wt_elim_cases})*})
+apply (tactic {*ALLGOALS (eresolve_tac @{context} @{thms wt_elim_cases})*})
 apply (simp_all (no_asm_use) split del: split_if_asm)
 apply (erule_tac [12] V = "All ?P" in thin_rl) (* Call *)
 apply (blast del: equalityCE dest: sym [THEN trans])+