doc-src/TutorialI/Protocol/Public.thy
changeset 32149 ef59550a55d3
parent 30608 d9805c5b5d2e
child 32960 69916a850301
--- a/doc-src/TutorialI/Protocol/Public.thy	Thu Jul 23 18:44:08 2009 +0200
+++ b/doc-src/TutorialI/Protocol/Public.thy	Thu Jul 23 18:44:09 2009 +0200
@@ -154,7 +154,7 @@
 ML {*
 fun possibility_tac ctxt =
     REPEAT (*omit used_Says so that Nonces start from different traces!*)
-    (ALLGOALS (simp_tac (local_simpset_of ctxt delsimps [used_Says]))
+    (ALLGOALS (simp_tac (simpset_of ctxt delsimps [used_Says]))
      THEN
      REPEAT_FIRST (eq_assume_tac ORELSE' 
                    resolve_tac [refl, conjI, @{thm Nonce_supply}]));