src/HOL/Library/Prefix_Order.thy
changeset 60500 903bb1495239
parent 58881 b9556a055632
child 60679 ade12ef2773c
equal deleted inserted replaced
60499:54a3db2ed201 60500:903bb1495239
     1 (*  Title:      HOL/Library/Prefix_Order.thy
     1 (*  Title:      HOL/Library/Prefix_Order.thy
     2     Author:     Tobias Nipkow and Markus Wenzel, TU Muenchen
     2     Author:     Tobias Nipkow and Markus Wenzel, TU Muenchen
     3 *)
     3 *)
     4 
     4 
     5 section {* Prefix order on lists as order class instance *}
     5 section \<open>Prefix order on lists as order class instance\<close>
     6 
     6 
     7 theory Prefix_Order
     7 theory Prefix_Order
     8 imports Sublist
     8 imports Sublist
     9 begin
     9 begin
    10 
    10