src/Sequents/LK.thy
changeset 55233 3229614ca9c5
parent 55230 cb5ef74b32f9
child 59498 50b60f501b05
--- a/src/Sequents/LK.thy	Sat Feb 01 18:17:13 2014 +0100
+++ b/src/Sequents/LK.thy	Sat Feb 01 18:22:38 2014 +0100
@@ -175,7 +175,7 @@
   assumes p1: "|- P <-> P'"
     and p2: "|- P' ==> |- Q <-> Q'"
   shows "|- (P-->Q) <-> (P'-->Q')"
-  apply (tactic {* lemma_tac @{thm p1} 1 *})
+  apply (lem p1)
   apply safe
    apply (tactic {*
      REPEAT (rtac @{thm cut} 1 THEN
@@ -188,7 +188,7 @@
   assumes p1: "|- P <-> P'"
     and p2: "|- P' ==> |- Q <-> Q'"
   shows "|- (P&Q) <-> (P'&Q')"
-  apply (tactic {* lemma_tac @{thm p1} 1 *})
+  apply (lem p1)
   apply safe
    apply (tactic {*
      REPEAT (rtac @{thm cut} 1 THEN
@@ -221,12 +221,12 @@
   done
 
 lemma if_cancel: "|- (if P then x else x) = x"
-  apply (tactic {* lemma_tac @{thm split_if} 1 *})
+  apply (lem split_if)
   apply fast
   done
 
 lemma if_eq_cancel: "|- (if x=y then y else x) = x"
-  apply (tactic {* lemma_tac @{thm split_if} 1 *})
+  apply (lem split_if)
   apply safe
   apply (rule symL)
   apply (rule basic)