src/HOL/Auth/Yahalom_Bad.thy
changeset 69597 ff784d5a5bfb
parent 67613 ce654b0e6d69
child 76287 cdc14f94c754
--- a/src/HOL/Auth/Yahalom_Bad.thy	Sat Jan 05 17:00:43 2019 +0100
+++ b/src/HOL/Auth/Yahalom_Bad.thy	Sat Jan 05 17:24:33 2019 +0100
@@ -106,7 +106,7 @@
        YM4_analz_knows_Spy [THEN analz_into_parts]
 
 
-text\<open>Theorems of the form @{term "X \<notin> parts (knows Spy evs)"} imply 
+text\<open>Theorems of the form \<^term>\<open>X \<notin> parts (knows Spy evs)\<close> imply 
             that NOBODY sends messages containing X!\<close>
 
 text\<open>Spy never sees a good agent's shared key!\<close>
@@ -334,9 +334,9 @@
 txt\<open>Fake\<close>
 apply blast
 txt\<open>YM3: by \<open>new_keys_not_used\<close>, the message
-   @{term "Crypt K (Nonce NB)"} could not exist\<close>
+   \<^term>\<open>Crypt K (Nonce NB)\<close> could not exist\<close>
 apply (force dest!: Crypt_imp_keysFor)
-txt\<open>YM4: was @{term "Crypt K (Nonce NB)"} the very last message?
+txt\<open>YM4: was \<^term>\<open>Crypt K (Nonce NB)\<close> the very last message?
     If not, use the induction hypothesis\<close>
 apply (simp add: ex_disj_distrib)
 txt\<open>yes: apply unicity of session keys\<close>