src/HOL/Combinatorics/Permutations.thy
changeset 73623 5020054b3a16
parent 73621 b4b70d13c995
child 73648 1bd3463e30b8
equal deleted inserted replaced
73622:4dc3baf45d6a 73623:5020054b3a16
     5 
     5 
     6 theory Permutations
     6 theory Permutations
     7   imports
     7   imports
     8     "HOL-Library.Multiset"
     8     "HOL-Library.Multiset"
     9     "HOL-Library.Disjoint_Sets"
     9     "HOL-Library.Disjoint_Sets"
       
    10     Transposition
    10 begin
    11 begin
    11 
    12 
    12 subsection \<open>Auxiliary\<close>
    13 subsection \<open>Auxiliary\<close>
    13 
    14 
    14 abbreviation (input) fixpoints :: \<open>('a \<Rightarrow> 'a) \<Rightarrow> 'a set\<close>
    15 abbreviation (input) fixpoints :: \<open>('a \<Rightarrow> 'a) \<Rightarrow> 'a set\<close>