src/HOL/Orderings.thy
changeset 18702 7dc7dcd63224
parent 17876 b9c92f384109
child 18851 9502ce541f01
equal deleted inserted replaced
18701:98e6a0a011f3 18702:7dc7dcd63224
   701 
   701 
   702   Alternatively, one can use "declare xtrans [trans]" and then
   702   Alternatively, one can use "declare xtrans [trans]" and then
   703   leave out the "(xtrans)" above.
   703   leave out the "(xtrans)" above.
   704 *)
   704 *)
   705 
   705 
       
   706 subsection {* Code generator setup *}
       
   707 
       
   708 code_alias
       
   709   "op <=" "Orderings.op_le"
       
   710   "op <" "Orderings.op_lt"
       
   711 
   706 end
   712 end