src/HOL/Auth/KerberosIV_Gets.thy
changeset 59807 22bc39064290
parent 58889 5b7a9633cfa8
child 61830 4f5ab843cf5b
--- a/src/HOL/Auth/KerberosIV_Gets.thy	Wed Mar 25 10:41:53 2015 +0100
+++ b/src/HOL/Auth/KerberosIV_Gets.thy	Wed Mar 25 10:44:57 2015 +0100
@@ -1238,11 +1238,12 @@
 txt{*K5. Not clear how this step could be integrated with the main
        simplification step. Done in KerberosV.thy*}
 apply clarify
-apply (erule_tac V = "Says Aa Tgs ?X \<in> set ?evs" in thin_rl)
+apply (erule_tac V = "Says Aa Tgs X \<in> set evs" for X evs in thin_rl)
 apply (frule Gets_imp_knows_Spy [THEN parts.Inj, THEN servK_notin_authKeysD])
 apply (assumption, assumption, blast, assumption)
 apply (simp add: analz_insert_freshK2)
-by (blast dest: Says_imp_spies [THEN parts.Inj] Key_unique_SesKey intro: less_SucI)
+apply (blast dest: Key_unique_SesKey intro: less_SucI)
+done
 
 
 text{* In the real world Tgs can't check wheter authK is secure! *}