src/HOL/Auth/Event.thy
changeset 67443 3abf6a722518
parent 63648 f9f3006a5579
child 67613 ce654b0e6d69
--- a/src/HOL/Auth/Event.thy	Tue Jan 16 09:12:16 2018 +0100
+++ b/src/HOL/Auth/Event.thy	Tue Jan 16 09:30:00 2018 +0100
@@ -72,7 +72,7 @@
                         Says A B X => parts {X} \<union> used evs
                       | Gets A X   => used evs
                       | Notes A X  => parts {X} \<union> used evs)"
-    \<comment>\<open>The case for @{term Gets} seems anomalous, but @{term Gets} always
+    \<comment> \<open>The case for @{term Gets} seems anomalous, but @{term Gets} always
         follows @{term Says} in real protocols.  Seems difficult to change.
         See \<open>Gets_correct\<close> in theory \<open>Guard/Extensions.thy\<close>.\<close>