diff -r bda7527ccf05 -r cc2d676d5395 src/Doc/Tutorial/Protocol/Event.thy --- a/src/Doc/Tutorial/Protocol/Event.thy Wed Dec 26 16:07:28 2018 +0100 +++ b/src/Doc/Tutorial/Protocol/Event.thy Wed Dec 26 16:25:20 2018 +0100 @@ -275,7 +275,7 @@ done -text\For proving @{text new_keys_not_used}\ +text\For proving \new_keys_not_used\\ lemma keysFor_parts_insert: "[| K \ keysFor (parts (insert X G)); X \ synth (analz H) |] ==> K \ keysFor (parts (G \ H)) | Key (invKey K) \ parts H" @@ -350,29 +350,29 @@ text \ The system's behaviour is formalized as a set of traces of -\emph{events}. The most important event, @{text "Says A B X"}, expresses +\emph{events}. The most important event, \Says A B X\, expresses $A\to B : X$, which is the attempt by~$A$ to send~$B$ the message~$X$. A trace is simply a list, constructed in reverse -using~@{text "#"}. Other event types include reception of messages (when +using~\#\. Other event types include reception of messages (when we want to make it explicit) and an agent's storing a fact. Sometimes the protocol requires an agent to generate a new nonce. The probability that a 20-byte random number has appeared before is effectively zero. To formalize this important property, the set @{term "used evs"} -denotes the set of all items mentioned in the trace~@{text evs}. -The function @{text used} has a straightforward -recursive definition. Here is the case for @{text Says} event: +denotes the set of all items mentioned in the trace~\evs\. +The function \used\ has a straightforward +recursive definition. Here is the case for \Says\ event: @{thm [display,indent=5] used_Says [no_vars]} -The function @{text knows} formalizes an agent's knowledge. Mostly we only +The function \knows\ formalizes an agent's knowledge. Mostly we only care about the spy's knowledge, and @{term "knows Spy evs"} is the set of items -available to the spy in the trace~@{text evs}. Already in the empty trace, +available to the spy in the trace~\evs\. Already in the empty trace, the spy starts with some secrets at his disposal, such as the private keys -of compromised users. After each @{text Says} event, the spy learns the +of compromised users. After each \Says\ event, the spy learns the message that was sent: @{thm [display,indent=5] knows_Spy_Says [no_vars]} Combinations of functions express other important -sets of messages derived from~@{text evs}: +sets of messages derived from~\evs\: \begin{itemize} \item @{term "analz (knows Spy evs)"} is everything that the spy could learn by decryption