src/HOL/TLA/Action.thy
changeset 30528 7173bf123335
parent 27104 791607529f6d
child 35108 e384e27c229f
--- a/src/HOL/TLA/Action.thy	Sun Mar 15 15:59:44 2009 +0100
+++ b/src/HOL/TLA/Action.thy	Sun Mar 15 15:59:44 2009 +0100
@@ -124,12 +124,9 @@
     | _ => th;
 *}
 
-setup {*
-  Attrib.add_attributes [
-    ("action_unlift", Attrib.no_args (Thm.rule_attribute (K action_unlift)), ""),
-    ("action_rewrite", Attrib.no_args (Thm.rule_attribute (K action_rewrite)), ""),
-    ("action_use", Attrib.no_args (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 =========================== *)