src/HOL/Library/Perm.thy
changeset 70335 9bd8c16b6627
parent 68406 6beb45f6cf67
child 72302 d7d90ed4c74e
equal deleted inserted replaced
70334:bba46912379e 70335:9bd8c16b6627
    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" ("(\<langle>$\<rangle>)")
       
    31 
    30 
    32 lemma bij_apply [simp]:
    31 lemma bij_apply [simp]:
    33   "bij (apply f)"
    32   "bij (apply f)"
    34   using "apply" [of f] by simp
    33   using "apply" [of f] by simp
    35 
    34 
   802 bundle permutation_syntax
   801 bundle permutation_syntax
   803 begin
   802 begin
   804   notation swap       ("\<langle>_\<leftrightarrow>_\<rangle>")
   803   notation swap       ("\<langle>_\<leftrightarrow>_\<rangle>")
   805   notation cycle      ("\<langle>_\<rangle>")
   804   notation cycle      ("\<langle>_\<rangle>")
   806   notation "apply"    (infixl "\<langle>$\<rangle>" 999)
   805   notation "apply"    (infixl "\<langle>$\<rangle>" 999)
   807   no_notation "apply" ("(\<langle>$\<rangle>)")
       
   808 end
   806 end
   809 
   807 
   810 unbundle no_permutation_syntax
   808 unbundle no_permutation_syntax
   811 
   809 
   812 end
   810 end