# HG changeset patch # User berghofe # Date 1185195896 -7200 # Node ID 6a98d0826dafc99d22d4fa3254ae6792ef589ac1 # Parent efee34ff4764096bd55bf8f548ba6a68c401c601 Tuned. diff -r efee34ff4764 -r 6a98d0826daf doc-src/TutorialI/Protocol/Message.thy --- a/doc-src/TutorialI/Protocol/Message.thy Mon Jul 23 14:39:21 2007 +0200 +++ b/doc-src/TutorialI/Protocol/Message.thy Mon Jul 23 15:04:56 2007 +0200 @@ -602,7 +602,7 @@ | MPair [intro]: "\X \ synth H; Y \ synth H\ \ \X,Y\ \ synth H" | Crypt [intro]: - "\X \ synth H; Key(K) \ H\ \ Crypt K X \ synth H" + "\X \ synth H; Key K \ H\ \ Crypt K X \ synth H" (*<*) lemma synth_mono: "G\H ==> synth(G) \ synth(H)" by (auto, erule synth.induct, auto) diff -r efee34ff4764 -r 6a98d0826daf doc-src/TutorialI/Protocol/document/Message.tex --- a/doc-src/TutorialI/Protocol/document/Message.tex Mon Jul 23 14:39:21 2007 +0200 +++ b/doc-src/TutorialI/Protocol/document/Message.tex Mon Jul 23 15:04:56 2007 +0200 @@ -1123,7 +1123,7 @@ \ \ {\isacharbar}\ MPair\ \ {\isacharbrackleft}intro{\isacharbrackright}{\isacharcolon}\isanewline \ \ \ \ \ \ \ \ \ \ \ \ \ \ {\isachardoublequoteopen}{\isasymlbrakk}X\ {\isasymin}\ synth\ H{\isacharsemicolon}\ \ Y\ {\isasymin}\ synth\ H{\isasymrbrakk}\ {\isasymLongrightarrow}\ {\isasymlbrace}X{\isacharcomma}Y{\isasymrbrace}\ {\isasymin}\ synth\ H{\isachardoublequoteclose}\isanewline \ \ {\isacharbar}\ Crypt\ \ {\isacharbrackleft}intro{\isacharbrackright}{\isacharcolon}\isanewline -\ \ \ \ \ \ \ \ \ \ \ \ \ \ {\isachardoublequoteopen}{\isasymlbrakk}X\ {\isasymin}\ synth\ H{\isacharsemicolon}\ \ Key{\isacharparenleft}K{\isacharparenright}\ {\isasymin}\ H{\isasymrbrakk}\ {\isasymLongrightarrow}\ Crypt\ K\ X\ {\isasymin}\ synth\ H{\isachardoublequoteclose}% +\ \ \ \ \ \ \ \ \ \ \ \ \ \ {\isachardoublequoteopen}{\isasymlbrakk}X\ {\isasymin}\ synth\ H{\isacharsemicolon}\ \ Key\ K\ {\isasymin}\ H{\isasymrbrakk}\ {\isasymLongrightarrow}\ Crypt\ K\ X\ {\isasymin}\ synth\ H{\isachardoublequoteclose}% \isadelimproof % \endisadelimproof