src/Sequents/LK/Nat.thy
changeset 55228 901a6696cdd8
parent 51717 9e7d1c139569
child 55229 08f2ebb65078
--- a/src/Sequents/LK/Nat.thy	Sat Feb 01 00:32:32 2014 +0000
+++ b/src/Sequents/LK/Nat.thy	Sat Feb 01 17:56:03 2014 +0100
@@ -37,7 +37,7 @@
 lemma Suc_n_not_n: "|- Suc(k) ~= k"
   apply (rule_tac n = k in induct)
   apply (tactic {* simp_tac (put_simpset LK_ss @{context} addsimps @{thms Suc_neq_0}) 1 *})
-  apply (tactic {* fast_tac (LK_pack add_safes @{thms Suc_inject_rule}) 1 *})
+  apply (fast add!: Suc_inject_rule)
   done
 
 lemma add_0: "|- 0+n = n"