src/FOLP/FOLP.thy
changeset 59498 50b60f501b05
parent 58957 c9e744ea8a38
child 60754 02924903a6fd
--- a/src/FOLP/FOLP.thy	Tue Feb 10 14:29:36 2015 +0100
+++ b/src/FOLP/FOLP.thy	Tue Feb 10 14:48:26 2015 +0100
@@ -57,7 +57,7 @@
   shows "?p : R"
   apply (rule excluded_middle [THEN disjE])
    apply (tactic {* DEPTH_SOLVE (atac 1 ORELSE
-       resolve_tac [@{thm r1}, @{thm r2}, @{thm major} RS @{thm mp}] 1) *})
+       resolve_tac @{context} [@{thm r1}, @{thm r2}, @{thm major} RS @{thm mp}] 1) *})
   done
 
 (*Double negation law*)
@@ -81,8 +81,8 @@
   apply (unfold iff_def)
   apply (rule conjE)
   apply (tactic {* DEPTH_SOLVE_1 (etac @{thm impCE} 1 ORELSE
-      eresolve_tac [@{thm notE}, @{thm impE}] 1 THEN atac 1 ORELSE atac 1 ORELSE
-      resolve_tac [@{thm r1}, @{thm r2}] 1) *})+
+      eresolve_tac @{context} [@{thm notE}, @{thm impE}] 1 THEN atac 1 ORELSE atac 1 ORELSE
+      resolve_tac @{context} [@{thm r1}, @{thm r2}] 1) *})+
   done