src/HOL/Auth/KerberosIV_Gets.thy
changeset 67443 3abf6a722518
parent 61830 4f5ab843cf5b
child 67613 ce654b0e6d69
--- a/src/HOL/Auth/KerberosIV_Gets.thy	Tue Jan 16 09:12:16 2018 +0100
+++ b/src/HOL/Auth/KerberosIV_Gets.thy	Tue Jan 16 09:30:00 2018 +0100
@@ -18,7 +18,7 @@
 
 axiomatization where
   Tgs_not_bad [iff]: "Tgs \<notin> bad"
-   \<comment>\<open>Tgs is secure --- we already know that Kas is secure\<close>
+   \<comment> \<open>Tgs is secure --- we already know that Kas is secure\<close>
 
 definition
  (* authKeys are those contained in an authTicket *)
@@ -1057,7 +1057,7 @@
         add: analz_image_freshK_simps AKcryptSK_Says shrK_not_AKcryptSK
              Oops2_not_AKcryptSK Auth_fresh_not_AKcryptSK
        Serv_fresh_not_AKcryptSK Says_Tgs_AKcryptSK Spy_analz_shrK)
-  \<comment>\<open>18 seconds on a 1.8GHz machine??\<close>
+  \<comment> \<open>18 seconds on a 1.8GHz machine??\<close>
 txt\<open>Fake\<close> 
 apply spy_analz
 txt\<open>Reception\<close>
@@ -1211,7 +1211,7 @@
 apply (erule rev_mp)
 apply (erule kerbIV_gets.induct)
 apply (rule_tac [10] impI)+
-  \<comment>\<open>The Oops1 case is unusual: must simplify
+  \<comment> \<open>The Oops1 case is unusual: must simplify
     @{term "Authkey \<notin> analz (spies (ev#evs))"}, not letting
    \<open>analz_mono_contra\<close> weaken it to
    @{term "Authkey \<notin> analz (spies evs)"},