src/CCL/Type.thy
changeset 51717 9e7d1c139569
parent 42814 5af15f1e2ef6
child 52143 36ffe23b25f8
--- a/src/CCL/Type.thy	Tue Apr 16 17:54:14 2013 +0200
+++ b/src/CCL/Type.thy	Thu Apr 18 17:07:01 2013 +0200
@@ -130,7 +130,7 @@
   SUBPROOF (fn {context = ctxt, prems = major :: prems, ...} =>
     resolve_tac ([major] RL top_crls) 1 THEN
     REPEAT_SOME (eresolve_tac (crls @ [@{thm exE}, @{thm bexE}, @{thm conjE}, @{thm disjE}])) THEN
-    ALLGOALS (asm_simp_tac (simpset_of ctxt)) THEN
+    ALLGOALS (asm_simp_tac ctxt) THEN
     ALLGOALS (ares_tac (prems RL [@{thm lem}]) ORELSE' etac @{thm bspec}) THEN
     safe_tac (ctxt addSIs prems))
 *}
@@ -415,7 +415,7 @@
 ML {*
 fun genIs_tac ctxt genXH gen_mono =
   rtac (genXH RS @{thm iffD2}) THEN'
-  simp_tac (simpset_of ctxt) THEN'
+  simp_tac ctxt THEN'
   TRY o fast_tac
     (ctxt addIs [genXH RS @{thm iffD2}, gen_mono RS @{thm coinduct3_mono_lemma} RS @{thm lfpI}])
 *}
@@ -498,7 +498,7 @@
  SELECT_GOAL
    (TRY (safe_tac ctxt) THEN
     resolve_tac ((rews @ [@{thm refl}]) RL ((rews @ [@{thm refl}]) RL [@{thm ssubst_pair}])) i THEN
-    ALLGOALS (simp_tac (simpset_of ctxt)) THEN
+    ALLGOALS (simp_tac ctxt) THEN
     ALLGOALS EQgen_raw_tac) i
 *}