Nominal-General/Nominal2_Eqvt.thy
changeset 2479 a9b6a00b1ba0
parent 2470 bdb1eab47161
child 2565 6bf332360510
equal deleted inserted replaced
2478:9b673588244a 2479:a9b6a00b1ba0
    72  {* pushes permutations inside, raises an error if it cannot solve all permutations. *}
    72  {* pushes permutations inside, raises an error if it cannot solve all permutations. *}
    73 
    73 
    74 (* the normal version of this lemma would cause loops *)
    74 (* the normal version of this lemma would cause loops *)
    75 lemma permute_eqvt_raw[eqvt_raw]:
    75 lemma permute_eqvt_raw[eqvt_raw]:
    76   shows "p \<bullet> permute \<equiv> permute"
    76   shows "p \<bullet> permute \<equiv> permute"
    77 apply(simp add: expand_fun_eq permute_fun_def)
    77 apply(simp add: fun_eq_iff permute_fun_def)
    78 apply(subst permute_eqvt)
    78 apply(subst permute_eqvt)
    79 apply(simp)
    79 apply(simp)
    80 done
    80 done
    81 
    81 
    82 section {* Logical Operators *}
    82 section {* Logical Operators *}