equal
deleted
inserted
replaced
258 should plug in only "very safe" rules that can be applied blindly. |
258 should plug in only "very safe" rules that can be applied blindly. |
259 Note that it applies whatever simplifications are currently active. |
259 Note that it applies whatever simplifications are currently active. |
260 *) |
260 *) |
261 fun action_simp_tac ctxt intros elims = |
261 fun action_simp_tac ctxt intros elims = |
262 asm_full_simp_tac |
262 asm_full_simp_tac |
263 (ctxt setloop (fn _ => (resolve_tac ctxt ((map (action_use ctxt) intros) |
263 (ctxt |> Simplifier.set_loop (fn _ => (resolve_tac ctxt ((map (action_use ctxt) intros) |
264 @ [refl,impI,conjI,@{thm actionI},@{thm intI},allI])) |
264 @ [refl,impI,conjI,@{thm actionI},@{thm intI},allI])) |
265 ORELSE' (eresolve_tac ctxt ((map (action_use ctxt) elims) |
265 ORELSE' (eresolve_tac ctxt ((map (action_use ctxt) elims) |
266 @ [conjE,disjE,exE])))); |
266 @ [conjE,disjE,exE])))); |
267 \<close> |
267 \<close> |
268 |
268 |