src/HOL/Auth/NS_Public.thy
changeset 11366 b42287eb20cf
parent 11230 756c5034f08b
child 13507 febb8e5d2a9d
--- a/src/HOL/Auth/NS_Public.thy	Sat Jun 09 08:42:29 2001 +0200
+++ b/src/HOL/Auth/NS_Public.thy	Sat Jun 09 08:43:38 2001 +0200
@@ -19,8 +19,8 @@
          (*The spy MAY say anything he CAN say.  We do not expect him to
            invent new nonces here, but he can also use NS1.  Common to
            all similar protocols.*)
-   Fake: "\<lbrakk>evs \<in> ns_public;  X \<in> synth (analz (spies evs))\<rbrakk>
-          \<Longrightarrow> Says Spy B X  # evs \<in> ns_public"
+   Fake: "\<lbrakk>evsf \<in> ns_public;  X \<in> synth (analz (spies evsf))\<rbrakk>
+          \<Longrightarrow> Says Spy B X  # evsf \<in> ns_public"
 
          (*Alice initiates a protocol run, sending a nonce to Bob*)
    NS1:  "\<lbrakk>evs1 \<in> ns_public;  Nonce NA \<notin> used evs1\<rbrakk>