src/HOL/Auth/NS_Public.thy
changeset 61830 4f5ab843cf5b
parent 58889 5b7a9633cfa8
child 76297 e7f9e5b3a36a
--- a/src/HOL/Auth/NS_Public.thy	Thu Dec 10 21:31:24 2015 +0100
+++ b/src/HOL/Auth/NS_Public.thy	Thu Dec 10 21:39:33 2015 +0100
@@ -6,7 +6,7 @@
 Version incorporating Lowe's fix (inclusion of B's identity in round 2).
 *)
 
-section{*Verifying the Needham-Schroeder-Lowe Public-Key Protocol*}
+section\<open>Verifying the Needham-Schroeder-Lowe Public-Key Protocol\<close>
 
 theory NS_Public imports Public begin
 
@@ -63,7 +63,7 @@
       "evs \<in> ns_public \<Longrightarrow> (Key (priEK A) \<in> analz (spies evs)) = (A \<in> bad)"
 by auto
 
-subsection{*Authenticity properties obtained from NS2*}
+subsection\<open>Authenticity properties obtained from NS2\<close>
 
 
 (*It is impossible to re-use a nonce in both NS1 and NS2, provided the nonce
@@ -135,7 +135,7 @@
 done
 
 
-subsection{*Authenticity properties obtained from NS2*}
+subsection\<open>Authenticity properties obtained from NS2\<close>
 
 (*Unicity for NS2: nonce NB identifies nonce NA and agents A, B 
   [unicity of B makes Lowe's fix work]
@@ -180,7 +180,7 @@
       \<Longrightarrow> Says A B (Crypt (pubEK B) (Nonce NB)) \<in> set evs"
 by (blast intro: B_trusts_NS3_lemma)
 
-subsection{*Overall guarantee for B*}
+subsection\<open>Overall guarantee for B\<close>
 
 (*If NS3 has been sent and the nonce NB agrees with the nonce B joined with
   NA, then A initiated the run using NA.*)