src/HOL/Bali/AxSem.thy
changeset 23894 1a4167d761ac
parent 23747 b07cff284683
child 24019 67bde7cfcf10
--- a/src/HOL/Bali/AxSem.thy	Sat Jul 21 17:40:40 2007 +0200
+++ b/src/HOL/Bali/AxSem.thy	Sat Jul 21 23:25:00 2007 +0200
@@ -670,7 +670,7 @@
 lemma ax_thin [rule_format (no_asm)]: 
   "G,(A'::'a triple set)|\<turnstile>(ts::'a triple set) \<Longrightarrow> \<forall>A. A' \<subseteq> A \<longrightarrow> G,A|\<turnstile>ts"
 apply (erule ax_derivs.induct)
-apply                (tactic "ALLGOALS(EVERY'[Clarify_tac,REPEAT o smp_tac 1])")
+apply                (tactic "ALLGOALS(EVERY'[clarify_tac @{claset}, REPEAT o smp_tac 1])")
 apply                (rule ax_derivs.empty)
 apply               (erule (1) ax_derivs.insert)
 apply              (fast intro: ax_derivs.asm)
@@ -712,7 +712,7 @@
 apply  (rule ax_derivs.conseq, clarify, tactic "smp_tac 3 1", blast(* unused *))
 (*37 subgoals*)
 apply (tactic {* TRYALL (resolve_tac ((funpow 5 tl) (thms "ax_derivs.intros")) 
-                   THEN_ALL_NEW Fast_tac) *})
+                   THEN_ALL_NEW fast_tac @{claset}) *})
 (*1 subgoal*)
 apply (clarsimp simp add: subset_mtriples_iff)
 apply (rule ax_derivs.Methd)