src/HOL/Auth/Kerberos_BAN_Gets.thy
changeset 44890 22f665a2e91c
parent 39251 8756b44582e2
child 55417 01fbfb60c33e
equal deleted inserted replaced
44889:340df9f3491f 44890:22f665a2e91c
   286 apply auto
   286 apply auto
   287 txt{*Two subcases of Message 2. Subcase: used before*}
   287 txt{*Two subcases of Message 2. Subcase: used before*}
   288 apply (blast dest: used_evs_rev [THEN equalityD2, THEN contra_subsetD] 
   288 apply (blast dest: used_evs_rev [THEN equalityD2, THEN contra_subsetD] 
   289                    used_takeWhile_used)
   289                    used_takeWhile_used)
   290 txt{*subcase: CT before*}
   290 txt{*subcase: CT before*}
   291 apply (fastsimp dest!: set_evs_rev [THEN equalityD2, THEN contra_subsetD, THEN takeWhile_void])
   291 apply (fastforce dest!: set_evs_rev [THEN equalityD2, THEN contra_subsetD, THEN takeWhile_void])
   292 done
   292 done
   293 
   293 
   294 
   294 
   295 text{*If the encrypted message appears then it originated with the Server
   295 text{*If the encrypted message appears then it originated with the Server
   296   PROVIDED that A is NOT compromised!
   296   PROVIDED that A is NOT compromised!