src/CCL/Type.thy
changeset 32149 ef59550a55d3
parent 32010 cb1a1c94b4cd
child 32153 a0e57fb1b930
--- a/src/CCL/Type.thy	Thu Jul 23 18:44:08 2009 +0200
+++ b/src/CCL/Type.thy	Thu Jul 23 18:44:09 2009 +0200
@@ -132,10 +132,10 @@
   fun mk_ncanT_tac ctxt defs top_crls crls s = prove_goalw (ProofContext.theory_of ctxt) defs s
     (fn major::prems => [(resolve_tac ([major] RL top_crls) 1),
                          (REPEAT_SOME (eresolve_tac (crls @ [exE,bexE,conjE,disjE]))),
-                         (ALLGOALS (asm_simp_tac (local_simpset_of ctxt))),
+                         (ALLGOALS (asm_simp_tac (simpset_of ctxt))),
                          (ALLGOALS (ares_tac (prems RL [lemma]) ORELSE'
                                     etac bspec )),
-                         (safe_tac (local_claset_of ctxt addSIs prems))])
+                         (safe_tac (claset_of ctxt addSIs prems))])
 end
 *}
 
@@ -408,7 +408,7 @@
 
 fun mk_genIs thy defs genXH gen_mono s = prove_goalw thy defs s
       (fn prems => [rtac (genXH RS iffD2) 1,
-                    simp_tac (simpset_of thy) 1,
+                    simp_tac (global_simpset_of thy) 1,
                     TRY (fast_tac (@{claset} addIs
                             ([genXH RS iffD2,gen_mono RS coinduct3_mono_lemma RS lfpI]
                              @ prems)) 1)])
@@ -442,7 +442,7 @@
    "[| <h,h'> : lfp(%x. POgen(x) Un R Un PO);  <t,t'> : lfp(%x. POgen(x) Un R Un PO) |] ==> <h$t,h'$t'> : POgen(lfp(%x. POgen(x) Un R Un PO))"];
 
 fun POgen_tac ctxt (rla,rlb) i =
-  SELECT_GOAL (safe_tac (local_claset_of ctxt)) i THEN
+  SELECT_GOAL (safe_tac (claset_of ctxt)) i THEN
   rtac (rlb RS (rla RS @{thm ssubst_pair})) i THEN
   (REPEAT (resolve_tac (POgenIs @ [@{thm PO_refl} RS (@{thm POgen_mono} RS ci3_AI)] @
     (POgenIs RL [@{thm POgen_mono} RS ci3_AgenI]) @ [@{thm POgen_mono} RS ci3_RI]) i));
@@ -481,9 +481,9 @@
 
 fun EQgen_tac ctxt rews i =
  SELECT_GOAL
-   (TRY (safe_tac (local_claset_of ctxt)) THEN
+   (TRY (safe_tac (claset_of ctxt)) THEN
     resolve_tac ((rews@[refl]) RL ((rews@[refl]) RL [@{thm ssubst_pair}])) i THEN
-    ALLGOALS (simp_tac (local_simpset_of ctxt)) THEN
+    ALLGOALS (simp_tac (simpset_of ctxt)) THEN
     ALLGOALS EQgen_raw_tac) i
 *}