src/HOL/SET_Protocol/Purchase.thy
changeset 42814 5af15f1e2ef6
parent 35703 29cb504abbb5
child 51798 ad3a241def73
equal deleted inserted replaced
42813:6c841fa92fa2 42814:5af15f1e2ef6
   482 method_setup valid_certificate_tac = {*
   482 method_setup valid_certificate_tac = {*
   483   Args.goal_spec >> (fn quant =>
   483   Args.goal_spec >> (fn quant =>
   484     K (SIMPLE_METHOD'' quant (fn i =>
   484     K (SIMPLE_METHOD'' quant (fn i =>
   485       EVERY [ftac @{thm Gets_certificate_valid} i,
   485       EVERY [ftac @{thm Gets_certificate_valid} i,
   486              assume_tac i, REPEAT (hyp_subst_tac i)])))
   486              assume_tac i, REPEAT (hyp_subst_tac i)])))
   487 *} ""
   487 *}
   488 
   488 
   489 
   489 
   490 subsection{*Proofs on Symmetric Keys*}
   490 subsection{*Proofs on Symmetric Keys*}
   491 
   491 
   492 text{*Nobody can have used non-existent keys!*}
   492 text{*Nobody can have used non-existent keys!*}