src/HOL/Auth/Recur.thy
changeset 69597 ff784d5a5bfb
parent 67613 ce654b0e6d69
child 76287 cdc14f94c754
--- a/src/HOL/Auth/Recur.thy	Sat Jan 05 17:00:43 2019 +0100
+++ b/src/HOL/Auth/Recur.thy	Sat Jan 05 17:24:33 2019 +0100
@@ -163,7 +163,7 @@
                                   [THEN respond.Cons, THEN respond.Cons]],
                      THEN recur.RA4, THEN recur.RA4])
 apply basic_possibility
-apply (tactic "DEPTH_SOLVE (swap_res_tac @{context} [refl, conjI, disjCI] 1)")
+apply (tactic "DEPTH_SOLVE (swap_res_tac \<^context> [refl, conjI, disjCI] 1)")
 done
 
 
@@ -396,8 +396,8 @@
 apply blast
 txt\<open>Inductive step of respond\<close>
 apply (intro allI conjI impI, simp_all)
-txt\<open>by unicity, either @{term "B=Aa"} or @{term "B=A'"}, a contradiction
-     if @{term "B \<in> bad"}\<close>   
+txt\<open>by unicity, either \<^term>\<open>B=Aa\<close> or \<^term>\<open>B=A'\<close>, a contradiction
+     if \<^term>\<open>B \<in> bad\<close>\<close>   
 apply (blast dest: unique_session_keys respond_certificate)
 apply (blast dest!: respond_certificate)
 apply (blast dest!: resp_analz_insert)