equal
deleted
inserted
replaced
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!*} |