| author | wenzelm |
| Tue, 02 Jul 2024 23:29:46 +0200 | |
| changeset 80482 | 2136ecf06a4c |
| 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 |