src/HOL/Combinatorics/Perm.thy
changeset 73623 5020054b3a16
parent 73622 4dc3baf45d6a
child 73648 1bd3463e30b8
equal deleted inserted replaced
73622:4dc3baf45d6a 73623:5020054b3a16
     1 (* Author: Florian Haftmann, TU Muenchen *)
     1 (* Author: Florian Haftmann, TU Muenchen *)
     2 
     2 
     3 section \<open>Permutations as abstract type\<close>
     3 section \<open>Permutations as abstract type\<close>
     4 
     4 
     5 theory Perm
     5 theory Perm
     6 imports Main
     6   imports
       
     7     Transposition
     7 begin
     8 begin
     8 
     9 
     9 text \<open>
    10 text \<open>
    10   This theory introduces basics about permutations, i.e. almost
    11   This theory introduces basics about permutations, i.e. almost
    11   everywhere fix bijections.  But it is by no means complete.
    12   everywhere fix bijections.  But it is by no means complete.