src/HOL/Library/Multiset.thy
changeset 14706 71590b7733b7
parent 14691 e1eedc8cad37
child 14722 8e739a6eaf11
equal deleted inserted replaced
14705:14b2c22a7e40 14706:71590b7733b7
     2     ID:         $Id$
     2     ID:         $Id$
     3     Author:     Tobias Nipkow, Markus Wenzel, and Lawrence C Paulson
     3     Author:     Tobias Nipkow, Markus Wenzel, and Lawrence C Paulson
     4     License:    GPL (GNU GENERAL PUBLIC LICENSE)
     4     License:    GPL (GNU GENERAL PUBLIC LICENSE)
     5 *)
     5 *)
     6 
     6 
     7 header {*
     7 header {* Multisets *}
     8  \title{Multisets}
       
     9  \author{Tobias Nipkow, Markus Wenzel, and Lawrence C Paulson}
       
    10 *}
       
    11 
     8 
    12 theory Multiset = Accessible_Part:
     9 theory Multiset = Accessible_Part:
    13 
    10 
    14 subsection {* The type of multisets *}
    11 subsection {* The type of multisets *}
    15 
    12