src/Sequents/LK/Hard_Quantifiers.thy
changeset 22896 1c2abcabea61
parent 21426 87ac12bed1ab
child 24178 4ff1dc2aa18d
--- a/src/Sequents/LK/Hard_Quantifiers.thy	Wed May 09 19:37:20 2007 +0200
+++ b/src/Sequents/LK/Hard_Quantifiers.thy	Wed May 09 19:37:21 2007 +0200
@@ -216,7 +216,7 @@
 
 text "Problem 48"
 lemma "|- (a=b | c=d) & (a=c | b=d) --> a=d | b=c"
-  by (tactic {* fast_tac (LK_pack add_safes [thm "subst"]) 1 *})
+  by (tactic {* fast_tac (LK_pack add_safes @{thms subst}) 1 *})
 
 text "Problem 50"
 lemma "|- (ALL x. P(a,x) | (ALL y. P(x,y))) --> (EX x. ALL y. P(x,y))"
@@ -225,16 +225,16 @@
 text "Problem 51"
 lemma "|- (EX z w. ALL x y. P(x,y) <->  (x=z & y=w)) -->   
          (EX z. ALL x. EX w. (ALL y. P(x,y) <-> y=w) <-> x=z)"
-  by (tactic {* fast_tac (LK_pack add_safes [thm "subst"]) 1 *})
+  by (tactic {* fast_tac (LK_pack add_safes @{thms subst}) 1 *})
 
 text "Problem 52"  (*Almost the same as 51. *)
 lemma "|- (EX z w. ALL x y. P(x,y) <->  (x=z & y=w)) -->
          (EX w. ALL y. EX z. (ALL x. P(x,y) <-> x=z) <-> y=w)"
-  by (tactic {* fast_tac (LK_pack add_safes [thm "subst"]) 1 *})
+  by (tactic {* fast_tac (LK_pack add_safes @{thms subst}) 1 *})
 
 text "Problem 56"
 lemma "|- (ALL x.(EX y. P(y) & x=f(y)) --> P(x)) <-> (ALL x. P(x) --> P(f(x)))"
-  by (tactic {* best_tac (LK_pack add_unsafes [thm "symL", thm "subst"]) 1 *})
+  by (tactic {* best_tac (LK_pack add_unsafes [@{thm symL}, @{thm subst}]) 1 *})
   (*requires tricker to orient the equality properly*)
 
 text "Problem 57"
@@ -244,7 +244,7 @@
 
 text "Problem 58!"
 lemma "|- (ALL x y. f(x)=g(y)) --> (ALL x y. f(f(x))=f(g(y)))"
-  by (tactic {* fast_tac (LK_pack add_safes [thm "subst"]) 1 *})
+  by (tactic {* fast_tac (LK_pack add_safes @{thms subst}) 1 *})
 
 text "Problem 59"
 (*Unification works poorly here -- the abstraction %sobj prevents efficient