src/HOL/Auth/Recur.thy
changeset 13956 8fe7e12290e1
parent 13935 4822d9597d1e
child 14200 d8598e24f8fa
--- a/src/HOL/Auth/Recur.thy	Mon May 05 15:55:56 2003 +0200
+++ b/src/HOL/Auth/Recur.thy	Mon May 05 18:22:01 2003 +0200
@@ -392,7 +392,8 @@
 apply blast
 txt{*Inductive step of respond*}
 apply (intro allI conjI impI, simp_all)
-txt{*by unicity, either B=Aa or B=A', a contradiction if B \<in> bad*}   
+txt{*by unicity, either @{term "B=Aa"} or @{term "B=A'"}, a contradiction
+     if @{term "B \<in> bad"}*}   
 apply (blast dest: unique_session_keys respond_certificate)
 apply (blast dest!: respond_certificate)
 apply (blast dest!: resp_analz_insert)