src/HOL/Combinatorics/Combinatorics.thy
author haftmann
Wed, 05 May 2021 16:09:02 +0000
changeset 73623 5020054b3a16
parent 73622 4dc3baf45d6a
child 73648 1bd3463e30b8
permissions -rw-r--r--
tuned theory structure


section \<open>Basic combinatorics in Isabelle/HOL (and the Archive of Formal Proofs)\<close>

theory Combinatorics
imports
  Transposition
  Stirling
  Permutations
  List_Permutation
  Multiset_Permutations
  Cycles
  Perm
begin

end