src/HOL/NanoJava/AxSem.thy
changeset 23894 1a4167d761ac
parent 23755 1c4672d130b1
child 35431 8758fe1fc9f8
--- a/src/HOL/NanoJava/AxSem.thy	Sat Jul 21 17:40:40 2007 +0200
+++ b/src/HOL/NanoJava/AxSem.thy	Sat Jul 21 23:25:00 2007 +0200
@@ -153,7 +153,7 @@
   "(A' |\<turnstile>  C         \<longrightarrow> (\<forall>A. A' \<subseteq> A \<longrightarrow> A |\<turnstile>  C       )) \<and> 
    (A'  \<turnstile>\<^sub>e {P} e {Q} \<longrightarrow> (\<forall>A. A' \<subseteq> A \<longrightarrow> A  \<turnstile>\<^sub>e {P} e {Q}))"
 apply (rule hoare_ehoare.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 (blast intro: hoare_ehoare.Skip)
 apply (blast intro: hoare_ehoare.Comp)
 apply (blast intro: hoare_ehoare.Cond)