src/HOL/SET_Protocol/Public_SET.thy
changeset 67443 3abf6a722518
parent 63648 f9f3006a5579
child 67613 ce654b0e6d69
--- a/src/HOL/SET_Protocol/Public_SET.thy	Tue Jan 16 09:12:16 2018 +0100
+++ b/src/HOL/SET_Protocol/Public_SET.thy	Tue Jan 16 09:30:00 2018 +0100
@@ -21,7 +21,7 @@
 
 consts
   publicKey :: "[bool, agent] => key"
-    \<comment>\<open>the boolean is TRUE if a signing key\<close>
+    \<comment> \<open>the boolean is TRUE if a signing key\<close>
 
 abbreviation "pubEK == publicKey False"
 abbreviation "pubSK == publicKey True"
@@ -110,7 +110,7 @@
 
 specification (pan)
   inj_pan: "inj pan"
-  \<comment>\<open>No two agents have the same PAN\<close>
+  \<comment> \<open>No two agents have the same PAN\<close>
 (*<*)
    apply (rule exI [of _ "nat_of_agent"]) 
    apply (simp add: inj_on_def inj_nat_of_agent [THEN inj_eq]) 
@@ -120,7 +120,7 @@
 declare inj_pan [THEN inj_eq, iff]
 
 consts
-  XOR :: "nat*nat => nat"  \<comment>\<open>no properties are assumed of exclusive-or\<close>
+  XOR :: "nat*nat => nat"  \<comment> \<open>no properties are assumed of exclusive-or\<close>
 
 
 subsection\<open>Signature Primitives\<close>
@@ -170,19 +170,19 @@
 subsection\<open>Encryption Primitives\<close>
 
 definition EXcrypt :: "[key,key,msg,msg] => msg" where
-  \<comment>\<open>Extra Encryption\<close>
+  \<comment> \<open>Extra Encryption\<close>
     (*K: the symmetric key   EK: the public encryption key*)
     "EXcrypt K EK M m =
        \<lbrace>Crypt K \<lbrace>M, Hash m\<rbrace>, Crypt EK \<lbrace>Key K, m\<rbrace>\<rbrace>"
 
 definition EXHcrypt :: "[key,key,msg,msg] => msg" where
-  \<comment>\<open>Extra Encryption with Hashing\<close>
+  \<comment> \<open>Extra Encryption with Hashing\<close>
     (*K: the symmetric key   EK: the public encryption key*)
     "EXHcrypt K EK M m =
        \<lbrace>Crypt K \<lbrace>M, Hash m\<rbrace>, Crypt EK \<lbrace>Key K, m, Hash M\<rbrace>\<rbrace>"
 
 definition Enc :: "[key,key,key,msg] => msg" where
-  \<comment>\<open>Simple Encapsulation with SIGNATURE\<close>
+  \<comment> \<open>Simple Encapsulation with SIGNATURE\<close>
     (*SK: the sender's signing key
       K: the symmetric key
       EK: the public encryption key*)
@@ -190,7 +190,7 @@
        \<lbrace>Crypt K (sign SK M), Crypt EK (Key K)\<rbrace>"
 
 definition EncB :: "[key,key,key,msg,msg] => msg" where
-  \<comment>\<open>Encapsulation with Baggage.  Keys as above, and baggage b.\<close>
+  \<comment> \<open>Encapsulation with Baggage.  Keys as above, and baggage b.\<close>
     "EncB SK K EK M b =
        \<lbrace>Enc SK K EK \<lbrace>M, Hash b\<rbrace>, b\<rbrace>"
 
@@ -386,7 +386,7 @@
 text\<open>Reverse the normal simplification of "image" to build up (not break down)
   the set of keys.  Based on \<open>analz_image_freshK_ss\<close>, but simpler.\<close>
 lemmas analz_image_keys_simps =
-       simp_thms mem_simps \<comment>\<open>these two allow its use with \<open>only:\<close>\<close>
+       simp_thms mem_simps \<comment> \<open>these two allow its use with \<open>only:\<close>\<close>
        image_insert [THEN sym] image_Un [THEN sym] 
        rangeI symKeys_neq_imp_neq
        insert_Key_singleton insert_Key_image Un_assoc [THEN sym]