equal
deleted
inserted
replaced
159 THEN |
159 THEN |
160 REPEAT_FIRST (eq_assume_tac ORELSE' |
160 REPEAT_FIRST (eq_assume_tac ORELSE' |
161 resolve_tac [refl, conjI, @{thm Nonce_supply}])); |
161 resolve_tac [refl, conjI, @{thm Nonce_supply}])); |
162 *} |
162 *} |
163 |
163 |
164 method_setup possibility = {* Method.no_args (SIMPLE_METHOD possibility_tac) *} |
164 method_setup possibility = {* Scan.succeed (K (SIMPLE_METHOD possibility_tac)) *} |
165 "for proving possibility theorems" |
165 "for proving possibility theorems" |
166 |
166 |
167 end |
167 end |
168 (*>*) |
168 (*>*) |