src/HOL/Library/Perm.thy
changeset 64911 f0e07600de47
parent 63993 9c0ff0c12116
child 67399 eab6ce8368fa
equal deleted inserted replaced
64910:6108dddad9f0 64911:f0e07600de47
    10   This theory introduces basics about permutations, i.e. almost
    10   This theory introduces basics about permutations, i.e. almost
    11   everywhere fix bijections.  But it is by no means complete.
    11   everywhere fix bijections.  But it is by no means complete.
    12   Grieviously missing are cycles since these would require more
    12   Grieviously missing are cycles since these would require more
    13   elaboration, e.g. the concept of distinct lists equivalent
    13   elaboration, e.g. the concept of distinct lists equivalent
    14   under rotation, which maybe would also deserve its own theory.
    14   under rotation, which maybe would also deserve its own theory.
    15   But see theory @{text "src/HOL/ex/Perm_Fragments.thy"} for
    15   But see theory \<open>src/HOL/ex/Perm_Fragments.thy\<close> for
    16   fragments on that.
    16   fragments on that.
    17 \<close>
    17 \<close>
    18 
    18 
    19 subsection \<open>Abstract type of permutations\<close>
    19 subsection \<open>Abstract type of permutations\<close>
    20 
    20