src/HOL/Library/List_Prefix.thy
changeset 15140 322485b816ac
parent 15131 c69542757a4d
child 15355 0de05d104060
equal deleted inserted replaced
15139:58cd3404cf75 15140:322485b816ac
     4 *)
     4 *)
     5 
     5 
     6 header {* List prefixes and postfixes *}
     6 header {* List prefixes and postfixes *}
     7 
     7 
     8 theory List_Prefix
     8 theory List_Prefix
     9 import Main
     9 imports Main
    10 begin
    10 begin
    11 
    11 
    12 subsection {* Prefix order on lists *}
    12 subsection {* Prefix order on lists *}
    13 
    13 
    14 instance list :: (type) ord ..
    14 instance list :: (type) ord ..