| author | wenzelm | 
| Sat, 13 Aug 2022 14:45:36 +0200 | |
| changeset 75841 | 7c00d5266bf8 | 
| parent 73648 | 1bd3463e30b8 | 
| permissions | -rw-r--r-- | 
| 73477 | 1 | |
| 2 | section \<open>Basic combinatorics in Isabelle/HOL (and the Archive of Formal Proofs)\<close> | |
| 3 | ||
| 4 | theory Combinatorics | |
| 5 | imports | |
| 73623 | 6 | Transposition | 
| 73477 | 7 | Stirling | 
| 8 | Permutations | |
| 9 | List_Permutation | |
| 10 | Multiset_Permutations | |
| 11 | Cycles | |
| 73622 | 12 | Perm | 
| 73648 | 13 | Orbits | 
| 73477 | 14 | begin | 
| 15 | ||
| 16 | end |