src/HOL/Quotient_Examples/Lift_DList.thy
changeset 53013 3fbcfa911863
parent 49834 b27bbb021df1
child 55524 f41ef840f09d
equal deleted inserted replaced
53012:cb82606b8215 53013:3fbcfa911863
     1 (*  Title:      HOL/Quotient_Examples/Lift_DList.thy
     1 (*  Title:      HOL/Quotient_Examples/Lift_DList.thy
     2     Author:     Ondrej Kuncar
     2     Author:     Ondrej Kuncar
     3 *)
     3 *)
     4 
     4 
     5 theory Lift_DList
     5 theory Lift_DList
     6 imports Main "~~/src/HOL/Library/Quotient_List"
     6 imports Main
     7 begin
     7 begin
     8 
     8 
     9 subsection {* The type of distinct lists *}
     9 subsection {* The type of distinct lists *}
    10 
    10 
    11 typedef 'a dlist = "{xs::'a list. distinct xs}"
    11 typedef 'a dlist = "{xs::'a list. distinct xs}"