src/HOL/Quotient_Examples/FSet.thy
changeset 45990 b7b905b23b2a
parent 45605 a89b4bc311a5
child 45994 38a46e029784
equal deleted inserted replaced
45989:b39256df5f8a 45990:b7b905b23b2a
     4 
     4 
     5 Type of finite sets.
     5 Type of finite sets.
     6 *)
     6 *)
     7 
     7 
     8 theory FSet
     8 theory FSet
     9 imports "~~/src/HOL/Library/Quotient_List" "~~/src/HOL/Library/More_List"
     9 imports "~~/src/HOL/Library/Quotient_List"
    10 begin
    10 begin
    11 
    11 
    12 text {* 
    12 text {* 
    13   The type of finite sets is created by a quotient construction
    13   The type of finite sets is created by a quotient construction
    14   over lists. The definition of the equivalence:
    14   over lists. The definition of the equivalence: