src/CTT/ex/Elimination.thy
changeset 59498 50b60f501b05
parent 58977 9576b510f6a2
child 60770 240563fbf41d
--- a/src/CTT/ex/Elimination.thy	Tue Feb 10 14:29:36 2015 +0100
+++ b/src/CTT/ex/Elimination.thy	Tue Feb 10 14:48:26 2015 +0100
@@ -182,7 +182,7 @@
     and "\<And>z. z:A*B \<Longrightarrow> C(z) type"
   shows "?a : (SUM z:A*B. C(z)) --> (SUM u:A. SUM v:B. C(<u,v>))"
 apply (rule intr_rls)
-apply (tactic {* biresolve_tac safe_brls 2 *})
+apply (tactic {* biresolve_tac @{context} safe_brls 2 *})
 (*Now must convert assumption C(z) into antecedent C(<kd,ke>) *)
 apply (rule_tac [2] a = "y" in ProdE)
 apply (typechk assms)