src/Doc/Tutorial/Protocol/Public.thy
changeset 59498 50b60f501b05
parent 51717 9e7d1c139569
child 62392 747d36865c2c
equal deleted inserted replaced
59497:0c5cd369a643 59498:50b60f501b05
   160 fun possibility_tac ctxt =
   160 fun possibility_tac ctxt =
   161     REPEAT (*omit used_Says so that Nonces start from different traces!*)
   161     REPEAT (*omit used_Says so that Nonces start from different traces!*)
   162     (ALLGOALS (simp_tac (ctxt delsimps [used_Says]))
   162     (ALLGOALS (simp_tac (ctxt delsimps [used_Says]))
   163      THEN
   163      THEN
   164      REPEAT_FIRST (eq_assume_tac ORELSE' 
   164      REPEAT_FIRST (eq_assume_tac ORELSE' 
   165                    resolve_tac [refl, conjI, @{thm Nonce_supply}]));
   165                    resolve_tac ctxt [refl, conjI, @{thm Nonce_supply}]));
   166 *}
   166 *}
   167 
   167 
   168 method_setup possibility = {* Scan.succeed (SIMPLE_METHOD o possibility_tac) *}
   168 method_setup possibility = {* Scan.succeed (SIMPLE_METHOD o possibility_tac) *}
   169     "for proving possibility theorems"
   169     "for proving possibility theorems"
   170 
   170