src/HOL/Orderings.thy
changeset 30510 4120fc59dd85
parent 30298 abefe1dfadbb
child 30515 bca05b17b618
--- a/src/HOL/Orderings.thy	Fri Mar 13 19:53:09 2009 +0100
+++ b/src/HOL/Orderings.thy	Fri Mar 13 19:58:26 2009 +0100
@@ -398,7 +398,7 @@
 
 val setup =
   Method.add_methods
-    [("order", Method.ctxt_args (Method.SIMPLE_METHOD' o order_tac []), "transitivity reasoner")] #>
+    [("order", Method.ctxt_args (SIMPLE_METHOD' o order_tac []), "transitivity reasoner")] #>
   Attrib.add_attributes [("order", attribute, "theorems controlling transitivity reasoner")];
 
 end;