src/HOL/TLA/TLA.thy
changeset 42769 053b4b487085
parent 41529 ba60efa2fd08
child 42773 29042b3e7575
--- a/src/HOL/TLA/TLA.thy	Thu May 12 21:14:03 2011 +0200
+++ b/src/HOL/TLA/TLA.thy	Thu May 12 22:07:30 2011 +0200
@@ -607,6 +607,16 @@
        (ss addsimps [@{thm Init_stp}, @{thm Init_act}]) [] [@{thm squareE}])));
 *}
 
+method_setup invariant = {*
+  Method.sections Clasimp.clasimp_modifiers
+    >> (K (SIMPLE_METHOD' o inv_tac o clasimpset_of))
+*} ""
+
+method_setup auto_invariant = {*
+  Method.sections Clasimp.clasimp_modifiers
+    >> (K (SIMPLE_METHOD' o auto_inv_tac o simpset_of))
+*} ""
+
 lemma unless: "|- []($P --> P` | Q`) --> (stable P) | <>Q"
   apply (unfold dmd_def)
   apply (clarsimp dest!: BoxPrime [temp_use])