src/HOLCF/ex/Focus_ex.thy
changeset 37598 893dcabf0c04
parent 35916 d5c5fc1b993b
child 39159 0dec18004e75
--- a/src/HOLCF/ex/Focus_ex.thy	Mon Jun 28 15:32:13 2010 +0200
+++ b/src/HOLCF/ex/Focus_ex.thy	Mon Jun 28 15:32:17 2010 +0200
@@ -204,7 +204,7 @@
 done
 
 lemma lemma4: "is_g(g) --> def_g(g)"
-apply (tactic {* simp_tac (HOL_ss delsimps (thms "ex_simps" @ thms "all_simps")
+apply (tactic {* simp_tac (HOL_ss delsimps (@{thms HOL.ex_simps} @ @{thms HOL.all_simps})
   addsimps [thm "lemma1", thm "lemma2", thm "def_g_def"]) 1 *})
 apply (rule impI)
 apply (erule exE)