equal
deleted
inserted
replaced
152 |
152 |
153 (*Tactic for possibility theorems*) |
153 (*Tactic for possibility theorems*) |
154 ML {* |
154 ML {* |
155 fun possibility_tac ctxt = |
155 fun possibility_tac ctxt = |
156 REPEAT (*omit used_Says so that Nonces start from different traces!*) |
156 REPEAT (*omit used_Says so that Nonces start from different traces!*) |
157 (ALLGOALS (simp_tac (local_simpset_of ctxt delsimps [used_Says])) |
157 (ALLGOALS (simp_tac (simpset_of ctxt delsimps [used_Says])) |
158 THEN |
158 THEN |
159 REPEAT_FIRST (eq_assume_tac ORELSE' |
159 REPEAT_FIRST (eq_assume_tac ORELSE' |
160 resolve_tac [refl, conjI, @{thm Nonce_supply}])); |
160 resolve_tac [refl, conjI, @{thm Nonce_supply}])); |
161 *} |
161 *} |
162 |
162 |