Nominal/Abs.thy
changeset 2104 2205b572bc9b
parent 2092 c0ab7451b20d
child 2124 a17b25cb94a6
equal deleted inserted replaced
2103:e08e3c29dbc0 2104:2205b572bc9b
   758   using a
   758   using a
   759   unfolding alphas fresh_star_def
   759   unfolding alphas fresh_star_def
   760   by (simp_all add: fresh_plus_perm)
   760   by (simp_all add: fresh_plus_perm)
   761 
   761 
   762 
   762 
   763 lemma alpha_gen_eqvt(*[eqvt]*):
   763 lemma alpha_gen_eqvt[eqvt]:
   764   shows "(bs, x) \<approx>gen R f q (cs, y) \<Longrightarrow> (p \<bullet> bs, p \<bullet> x) \<approx>gen (p \<bullet> R) (p \<bullet> f) (p \<bullet> q) (p \<bullet> cs, p \<bullet> y)"
   764   shows "(bs, x) \<approx>gen R f q (cs, y) \<Longrightarrow> (p \<bullet> bs, p \<bullet> x) \<approx>gen (p \<bullet> R) (p \<bullet> f) (p \<bullet> q) (p \<bullet> cs, p \<bullet> y)"
   765   and   "(bs, x) \<approx>res R f q (cs, y) \<Longrightarrow> (p \<bullet> bs, p \<bullet> x) \<approx>res (p \<bullet> R) (p \<bullet> f) (p \<bullet> q) (p \<bullet> cs, p \<bullet> y)"
   765   and   "(bs, x) \<approx>res R f q (cs, y) \<Longrightarrow> (p \<bullet> bs, p \<bullet> x) \<approx>res (p \<bullet> R) (p \<bullet> f) (p \<bullet> q) (p \<bullet> cs, p \<bullet> y)"
   766   and   "(ds, x) \<approx>lst R f q (es, y) \<Longrightarrow> (p \<bullet> ds, p \<bullet> x) \<approx>lst (p \<bullet> R) (p \<bullet> f) (p \<bullet> q) (p \<bullet> es, p \<bullet> y)" 
   766   and   "(ds, x) \<approx>lst R f q (es, y) \<Longrightarrow> (p \<bullet> ds, p \<bullet> x) \<approx>lst (p \<bullet> R) (p \<bullet> f) (p \<bullet> q) (p \<bullet> es, p \<bullet> y)" 
   767   unfolding alphas
   767   unfolding alphas
   768   unfolding permute_eqvt[symmetric]
   768   unfolding permute_eqvt[symmetric]