src/HOL/Library/Permutations.thy
changeset 34102 d397496894c4
parent 33715 8cce3a34c122
child 36335 ceea7e15c04b
equal deleted inserted replaced
34101:d689f0b33047 34102:d397496894c4
    13 
    13 
    14 (* ------------------------------------------------------------------------- *)
    14 (* ------------------------------------------------------------------------- *)
    15 (* Transpositions.                                                           *)
    15 (* Transpositions.                                                           *)
    16 (* ------------------------------------------------------------------------- *)
    16 (* ------------------------------------------------------------------------- *)
    17 
    17 
    18 declare swap_self[simp]
       
    19 lemma swapid_sym: "Fun.swap a b id = Fun.swap b a id"
    18 lemma swapid_sym: "Fun.swap a b id = Fun.swap b a id"
    20   by (auto simp add: expand_fun_eq swap_def fun_upd_def)
    19   by (auto simp add: expand_fun_eq swap_def fun_upd_def)
    21 lemma swap_id_refl: "Fun.swap a a id = id" by simp
    20 lemma swap_id_refl: "Fun.swap a a id = id" by simp
    22 lemma swap_id_sym: "Fun.swap a b id = Fun.swap b a id"
    21 lemma swap_id_sym: "Fun.swap a b id = Fun.swap b a id"
    23   by (rule ext, simp add: swap_def)
    22   by (rule ext, simp add: swap_def)