src/HOL/Combinatorics/Combinatorics.thy
changeset 73477 1d8a79aa2a99
child 73622 4dc3baf45d6a
equal deleted inserted replaced
73476:6b480efe1bc3 73477:1d8a79aa2a99
       
     1 
       
     2 section \<open>Basic combinatorics in Isabelle/HOL (and the Archive of Formal Proofs)\<close>
       
     3 
       
     4 theory Combinatorics
       
     5 imports
       
     6   Stirling
       
     7   Permutations
       
     8   List_Permutation
       
     9   Multiset_Permutations
       
    10   Cycles
       
    11 begin
       
    12 
       
    13 end