src/Sequents/LK.thy
changeset 59498 50b60f501b05
parent 55233 3229614ca9c5
child 60754 02924903a6fd
--- a/src/Sequents/LK.thy	Tue Feb 10 14:29:36 2015 +0100
+++ b/src/Sequents/LK.thy	Tue Feb 10 14:48:26 2015 +0100
@@ -180,7 +180,7 @@
    apply (tactic {*
      REPEAT (rtac @{thm cut} 1 THEN
        DEPTH_SOLVE_1
-         (resolve_tac [@{thm thinL}, @{thm thinR}, @{thm p2} COMP @{thm monotonic}] 1) THEN
+         (resolve_tac @{context} [@{thm thinL}, @{thm thinR}, @{thm p2} COMP @{thm monotonic}] 1) THEN
            Cla.safe_tac @{context} 1) *})
   done
 
@@ -193,7 +193,7 @@
    apply (tactic {*
      REPEAT (rtac @{thm cut} 1 THEN
        DEPTH_SOLVE_1
-         (resolve_tac [@{thm thinL}, @{thm thinR}, @{thm p2} COMP @{thm monotonic}] 1) THEN
+         (resolve_tac @{context} [@{thm thinL}, @{thm thinR}, @{thm p2} COMP @{thm monotonic}] 1) THEN
            Cla.safe_tac @{context} 1) *})
   done