diff -r c8a2755bf220 -r ff784d5a5bfb src/HOL/SET_Protocol/Public_SET.thy --- a/src/HOL/SET_Protocol/Public_SET.thy Sat Jan 05 17:00:43 2019 +0100 +++ b/src/HOL/SET_Protocol/Public_SET.thy Sat Jan 05 17:24:33 2019 +0100 @@ -31,7 +31,7 @@ abbreviation "priSK A == invKey (pubSK A)" text\By freeness of agents, no two agents have the same key. Since - @{term "True\False"}, no agent has the same signing and encryption keys.\ + \<^term>\True\False\, no agent has the same signing and encryption keys.\ specification (publicKey) injective_publicKey: @@ -367,7 +367,7 @@ "for proving possibility theorems" -subsection\Specialized Rewriting for Theorems About @{term analz} and Image\ +subsection\Specialized Rewriting for Theorems About \<^term>\analz\ and Image\ lemma insert_Key_singleton: "insert (Key K) H = Key ` {K} \ H" by blast @@ -411,7 +411,7 @@ keysFor (insert A X) = keysFor (insert B X)" by auto -subsubsection\Special Simplification Rules for @{term signCert}\ +subsubsection\Special Simplification Rules for \<^term>\signCert\\ text\Avoids duplicating X and its components!\ lemma parts_insert_signCert: @@ -428,7 +428,7 @@ lemma keysFor_insert_signCert: "keysFor (insert (signCert K X) H) = keysFor H" by (simp add: signCert_def) -text\Controlled rewrite rules for @{term signCert}, just the definitions +text\Controlled rewrite rules for \<^term>\signCert\, just the definitions of the others. Encryption primitives are just expanded, despite their huge redundancy!\ lemmas abbrev_simps [simp] = @@ -477,7 +477,7 @@ by (unfold EXcrypt_def, blast) -subsection\Lemmas to Simplify Expressions Involving @{term analz}\ +subsection\Lemmas to Simplify Expressions Involving \<^term>\analz\\ lemma analz_knows_absorb: "Key K \ analz (knows Spy evs) @@ -511,7 +511,7 @@ "[|Key K \ parts {X}; Says A B X \ set evs|] ==> Key K \ used evs" by (blast intro: parts_trans dest!: Says_imp_knows_Spy [THEN parts.Inj]) -text\A useful rewrite rule with @{term analz_image_keys_simps}\ +text\A useful rewrite rule with \<^term>\analz_image_keys_simps\\ lemma Crypt_notin_image_Key: "Crypt K X \ Key ` KK" by auto