src/HOL/Auth/KerberosIV.thy
changeset 13507 febb8e5d2a9d
parent 11704 3c50a2cd6f00
child 14182 5f49f00fe084
--- a/src/HOL/Auth/KerberosIV.thy	Fri Aug 16 17:19:43 2002 +0200
+++ b/src/HOL/Auth/KerberosIV.thy	Sat Aug 17 14:55:08 2002 +0200
@@ -44,7 +44,7 @@
                       
  (* A is the true creator of X if she has sent X and X never appeared on
     the trace before this event. Recall that traces grow from head. *)
-  Issues :: [agent , agent, msg, event list] => bool ("_ Issues _ with _ on _")
+  Issues :: [agent, agent, msg, event list] => bool ("_ Issues _ with _ on _")
    "A Issues B with X on evs == 
       \\<exists>Y. Says A B Y \\<in> set evs & X \\<in> parts {Y} &
       X \\<notin> parts (spies (takeWhile (% z. z  \\<noteq> Says A B Y) (rev evs)))"