changeset 65552 | f533820e7248 |
parent 65342 | e32eb488c3a3 |
child 66486 | ffaaa83543b2 |
--- a/src/HOL/Library/Permutations.thy Sat Apr 22 12:52:55 2017 +0200 +++ b/src/HOL/Library/Permutations.thy Sat Apr 22 22:01:35 2017 +0200 @@ -5,7 +5,7 @@ section \<open>Permutations, both general and specifically on finite sets.\<close> theory Permutations - imports Binomial Multiset Disjoint_Sets + imports Multiset Disjoint_Sets begin subsection \<open>Transpositions\<close>