src/HOL/Library/Perm.thy
changeset 67399 eab6ce8368fa
parent 64911 f0e07600de47
child 68406 6beb45f6cf67
equal deleted inserted replaced
67398:5eb932e604a2 67399:eab6ce8368fa
    25 qed
    25 qed
    26 
    26 
    27 setup_lifting type_definition_perm
    27 setup_lifting type_definition_perm
    28 
    28 
    29 notation "apply" (infixl "\<langle>$\<rangle>" 999)
    29 notation "apply" (infixl "\<langle>$\<rangle>" 999)
    30 no_notation "apply" ("op \<langle>$\<rangle>")
    30 no_notation "apply" ("(\<langle>$\<rangle>)")
    31 
    31 
    32 lemma bij_apply [simp]:
    32 lemma bij_apply [simp]:
    33   "bij (apply f)"
    33   "bij (apply f)"
    34   using "apply" [of f] by simp
    34   using "apply" [of f] by simp
    35 
    35 
   802 bundle permutation_syntax
   802 bundle permutation_syntax
   803 begin
   803 begin
   804   notation swap       ("\<langle>_\<leftrightarrow>_\<rangle>")
   804   notation swap       ("\<langle>_\<leftrightarrow>_\<rangle>")
   805   notation cycle      ("\<langle>_\<rangle>")
   805   notation cycle      ("\<langle>_\<rangle>")
   806   notation "apply"    (infixl "\<langle>$\<rangle>" 999)
   806   notation "apply"    (infixl "\<langle>$\<rangle>" 999)
   807   no_notation "apply" ("op \<langle>$\<rangle>")
   807   no_notation "apply" ("(\<langle>$\<rangle>)")
   808 end
   808 end
   809 
   809 
   810 unbundle no_permutation_syntax
   810 unbundle no_permutation_syntax
   811 
   811 
   812 end
   812 end