diff -r c8a2755bf220 -r ff784d5a5bfb src/HOL/Metis_Examples/Message.thy --- a/src/HOL/Metis_Examples/Message.thy Sat Jan 05 17:00:43 2019 +0100 +++ b/src/HOL/Metis_Examples/Message.thy Sat Jan 05 17:24:33 2019 +0100 @@ -217,7 +217,7 @@ text\This allows \blast\ to simplify occurrences of - @{term "parts(G\H)"} in the assumption.\ + \<^term>\parts(G\H)\ in the assumption.\ lemmas in_parts_UnE = parts_Un [THEN equalityD1, THEN subsetD, THEN UnE] declare in_parts_UnE [elim!] @@ -461,8 +461,8 @@ text\Case analysis: either the message is secure, or it is not! Effective, but can cause subgoals to blow up! Use with \if_split\; apparently -\split_tac\ does not cope with patterns such as @{term"analz (insert -(Crypt K X) H)"}\ +\split_tac\ does not cope with patterns such as \<^term>\analz (insert +(Crypt K X) H)\\ lemma analz_Crypt_if [simp]: "analz (insert (Crypt K X) H) = (if (Key (invKey K) \ analz H) @@ -576,7 +576,7 @@ by (auto, erule synth.induct, auto) text\NO \Agent_synth\, as any Agent name can be synthesized. - The same holds for @{term Number}\ + The same holds for \<^term>\Number\\ inductive_cases Nonce_synth [elim!]: "Nonce n \ synth H" inductive_cases Key_synth [elim!]: "Key K \ synth H" inductive_cases Hash_synth [elim!]: "Hash X \ synth H"