src/HOL/TLA/Action.thy
changeset 42814 5af15f1e2ef6
parent 42793 88bee9f6eec7
child 47968 3119ad2b5ad3
--- a/src/HOL/TLA/Action.thy	Sun May 15 17:06:35 2011 +0200
+++ b/src/HOL/TLA/Action.thy	Sun May 15 17:45:53 2011 +0200
@@ -120,9 +120,9 @@
     | _ => th;
 *}
 
-attribute_setup action_unlift = {* Scan.succeed (Thm.rule_attribute (K action_unlift)) *} ""
-attribute_setup action_rewrite = {* Scan.succeed (Thm.rule_attribute (K action_rewrite)) *} ""
-attribute_setup action_use = {* Scan.succeed (Thm.rule_attribute (K action_use)) *} ""
+attribute_setup action_unlift = {* Scan.succeed (Thm.rule_attribute (K action_unlift)) *}
+attribute_setup action_rewrite = {* Scan.succeed (Thm.rule_attribute (K action_rewrite)) *}
+attribute_setup action_use = {* Scan.succeed (Thm.rule_attribute (K action_use)) *}
 
 
 (* =========================== square / angle brackets =========================== *)
@@ -283,7 +283,7 @@
 
 method_setup enabled = {*
   Attrib.thm >> (fn th => fn ctxt => SIMPLE_METHOD' (enabled_tac ctxt th))
-*} ""
+*}
 
 (* Example *)