src/HOL/Library/Permutations.thy
changeset 65552 f533820e7248
parent 65342 e32eb488c3a3
child 66486 ffaaa83543b2
equal deleted inserted replaced
65551:d164c4fc0d2c 65552:f533820e7248
     3 *)
     3 *)
     4 
     4 
     5 section \<open>Permutations, both general and specifically on finite sets.\<close>
     5 section \<open>Permutations, both general and specifically on finite sets.\<close>
     6 
     6 
     7 theory Permutations
     7 theory Permutations
     8   imports Binomial Multiset Disjoint_Sets
     8   imports Multiset Disjoint_Sets
     9 begin
     9 begin
    10 
    10 
    11 subsection \<open>Transpositions\<close>
    11 subsection \<open>Transpositions\<close>
    12 
    12 
    13 lemma swap_id_idempotent [simp]: "Fun.swap a b id \<circ> Fun.swap a b id = id"
    13 lemma swap_id_idempotent [simp]: "Fun.swap a b id \<circ> Fun.swap a b id = id"