src/HOL/Auth/Smartcard/EventSC.thy
changeset 67443 3abf6a722518
parent 66453 cc19f7ca2ed6
child 69597 ff784d5a5bfb
--- a/src/HOL/Auth/Smartcard/EventSC.thy	Tue Jan 16 09:12:16 2018 +0100
+++ b/src/HOL/Auth/Smartcard/EventSC.thy	Tue Jan 16 09:30:00 2018 +0100
@@ -95,7 +95,7 @@
                   | C_Gets C X   => used evs
                   | Outpts C A X  => parts{X} \<union> (used evs)
                   | A_Gets A X   => used evs)"
-    \<comment>\<open>@{term Gets} always follows @{term Says} in real protocols. 
+    \<comment> \<open>@{term Gets} always follows @{term Says} in real protocols. 
        Likewise, @{term C_Gets} will always have to follow @{term Inputs}
        and @{term A_Gets} will always have to follow @{term Outpts}\<close>