src/HOL/Orderings.thy
changeset 24867 e5b55d7be9bb
parent 24748 ee0a0eb6b738
child 24920 2a45e400fdad
--- a/src/HOL/Orderings.thy	Sat Oct 06 16:41:22 2007 +0200
+++ b/src/HOL/Orderings.thy	Sat Oct 06 16:50:04 2007 +0200
@@ -346,7 +346,7 @@
     (Context.cases (print_structures o ProofContext.init) print_structures)
     (print_structures o Proof.context_of));
 
-val printP =
+val _ =
   OuterSyntax.improper_command "print_orders"
     "print order structures available to transitivity reasoner" OuterKeyword.diag
     (Scan.succeed (Toplevel.no_timing o print));
@@ -354,11 +354,10 @@
 
 (** Setup **)
 
-val setup = let val _ = OuterSyntax.add_parsers [printP] in
-    Method.add_methods [("order", Method.ctxt_args (Method.SIMPLE_METHOD' o order_tac []),
-      "normalisation of algebraic structure")] #>
-    Attrib.add_attributes [("order", attribute, "theorems controlling transitivity reasoner")]
-  end;
+val setup =
+  Method.add_methods
+    [("order", Method.ctxt_args (Method.SIMPLE_METHOD' o order_tac []), "transitivity reasoner")] #>
+  Attrib.add_attributes [("order", attribute, "theorems controlling transitivity reasoner")];
 
 end;