src/HOL/TLA/Action.thy
changeset 59498 50b60f501b05
parent 58889 5b7a9633cfa8
child 59582 0fbed69ff081
--- a/src/HOL/TLA/Action.thy	Tue Feb 10 14:29:36 2015 +0100
+++ b/src/HOL/TLA/Action.thy	Tue Feb 10 14:48:26 2015 +0100
@@ -263,9 +263,9 @@
 *)
 fun action_simp_tac ctxt intros elims =
     asm_full_simp_tac
-         (ctxt setloop (fn _ => (resolve_tac ((map (action_use ctxt) intros)
+         (ctxt setloop (fn _ => (resolve_tac ctxt ((map (action_use ctxt) intros)
                                     @ [refl,impI,conjI,@{thm actionI},@{thm intI},allI]))
-                      ORELSE' (eresolve_tac ((map (action_use ctxt) elims)
+                      ORELSE' (eresolve_tac ctxt ((map (action_use ctxt) elims)
                                              @ [conjE,disjE,exE]))));
 *}