src/Doc/Tutorial/Protocol/Message.thy
changeset 67443 3abf6a722518
parent 67406 23307fd33906
child 67613 ce654b0e6d69
--- a/src/Doc/Tutorial/Protocol/Message.thy	Tue Jan 16 09:12:16 2018 +0100
+++ b/src/Doc/Tutorial/Protocol/Message.thy	Tue Jan 16 09:30:00 2018 +0100
@@ -35,7 +35,7 @@
 type_synonym key = nat
 consts invKey :: "key \<Rightarrow> key"
 (*<*)
-consts all_symmetric :: bool        \<comment>\<open>true if all keys are symmetric\<close>
+consts all_symmetric :: bool        \<comment> \<open>true if all keys are symmetric\<close>
 
 specification (invKey)
   invKey [simp]: "invKey (invKey K) = K"
@@ -88,7 +88,7 @@
 
 
 definition keysFor :: "msg set => key set" where
-    \<comment>\<open>Keys useful to decrypt elements of a message set\<close>
+    \<comment> \<open>Keys useful to decrypt elements of a message set\<close>
   "keysFor H == invKey ` {K. \<exists>X. Crypt K X \<in> H}"