src/Pure/Pure.thy
changeset 55152 a56099a6447a
parent 55141 863b4f9f6bd7
child 55385 169e12bbf9a3
--- a/src/Pure/Pure.thy	Sun Jan 26 13:45:40 2014 +0100
+++ b/src/Pure/Pure.thy	Sun Jan 26 14:01:19 2014 +0100
@@ -175,10 +175,6 @@
   "Scan.lift (Parse.and_list1 (Scan.repeat Args.name)) >> Rule_Cases.params"
   "named rule parameters"
 
-attribute_setup standard =
-  "Scan.succeed (Thm.rule_attribute (K Drule.export_without_context))"
-  "result put into standard form (legacy)"
-
 attribute_setup rule_format = {*
   Scan.lift (Args.mode "no_asm")
     >> (fn true => Object_Logic.rule_format_no_asm | false => Object_Logic.rule_format)