src/HOL/Combinatorics/Combinatorics.thy
author wenzelm
Mon, 20 May 2024 15:43:51 +0200
changeset 80182 29f2b8ff84f3
parent 73648 1bd3463e30b8
permissions -rw-r--r--
proper support for "isabelle update -D DIR": avoid accidental exclusion of select_dirs (amending e5dafe9e120f);


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
  Orbits
begin

end