src/HOL/Auth/Message.thy
changeset 26342 0f65fa163304
parent 24122 fc7f857d33c8
child 26807 4cd176ea28dc
--- a/src/HOL/Auth/Message.thy	Wed Mar 19 22:47:39 2008 +0100
+++ b/src/HOL/Auth/Message.thy	Wed Mar 19 22:50:42 2008 +0100
@@ -847,8 +847,8 @@
   concerns  Crypt K X \<notin> Key`shrK`bad  and cannot be proved by rewriting
   alone.*)
 fun prove_simple_subgoals_tac i = 
-    force_tac (claset(), simpset() addsimps [@{thm image_eq_UN}]) i THEN
-    ALLGOALS Asm_simp_tac
+    CLASIMPSET' (fn (cs, ss) => force_tac (cs, ss addsimps [@{thm image_eq_UN}])) i THEN
+    ALLGOALS (SIMPSET' asm_simp_tac)
 
 (*Analysis of Fake cases.  Also works for messages that forward unknown parts,
   but this application is no longer necessary if analz_insert_eq is used.
@@ -886,7 +886,7 @@
        REPEAT (FIRSTGOAL (resolve_tac [allI,impI,notI,conjI,iffI])),
        DEPTH_SOLVE (atomic_spy_analz_tac (cs,ss) 1)]) i)
 
-fun spy_analz_tac i = gen_spy_analz_tac (claset(), simpset()) i
+val spy_analz_tac = CLASIMPSET' gen_spy_analz_tac;
 
 end
 *}