src/HOL/Library/Product_ord.thy
changeset 25594 43c718438f9f
parent 25571 c9e39eafc7a0
child 25691 8f8d83af100a
equal deleted inserted replaced
25593:0b0df6c8646a 25594:43c718438f9f
     4 *)
     4 *)
     5 
     5 
     6 header {* Order on product types *}
     6 header {* Order on product types *}
     7 
     7 
     8 theory Product_ord
     8 theory Product_ord
     9 imports Main
     9 imports PreList
    10 begin
    10 begin
    11 
    11 
    12 instantiation "*" :: (ord, ord) ord
    12 instantiation "*" :: (ord, ord) ord
    13 begin
    13 begin
    14 
    14