src/HOL/Library/Permutations.thy
changeset 30663 0b6aff7451b2
parent 30488 5c4c3a9e9102
child 32456 341c83339aeb
equal deleted inserted replaced
30662:396be15b95d5 30663:0b6aff7451b2
     3 *)
     3 *)
     4 
     4 
     5 header {* Permutations, both general and specifically on finite sets.*}
     5 header {* Permutations, both general and specifically on finite sets.*}
     6 
     6 
     7 theory Permutations
     7 theory Permutations
     8 imports Main Finite_Cartesian_Product Parity Fact
     8 imports Finite_Cartesian_Product Parity Fact Main
     9 begin
     9 begin
    10 
    10 
    11   (* Why should I import Main just to solve the Typerep problem! *)
    11   (* Why should I import Main just to solve the Typerep problem! *)
    12 
    12 
    13 definition permutes (infixr "permutes" 41) where
    13 definition permutes (infixr "permutes" 41) where