src/HOL/Orderings.thy
changeset 30515 bca05b17b618
parent 30510 4120fc59dd85
child 30528 7173bf123335
equal deleted inserted replaced
30514:9455ecc7796d 30515:bca05b17b618
   395 
   395 
   396 
   396 
   397 (** Setup **)
   397 (** Setup **)
   398 
   398 
   399 val setup =
   399 val setup =
   400   Method.add_methods
   400   Method.setup @{binding order} (Scan.succeed (SIMPLE_METHOD' o order_tac [])) "transitivity reasoner" #>
   401     [("order", Method.ctxt_args (SIMPLE_METHOD' o order_tac []), "transitivity reasoner")] #>
       
   402   Attrib.add_attributes [("order", attribute, "theorems controlling transitivity reasoner")];
   401   Attrib.add_attributes [("order", attribute, "theorems controlling transitivity reasoner")];
   403 
   402 
   404 end;
   403 end;
   405 
   404 
   406 *}
   405 *}