diff -r c123419a4eb0 -r b7423c6b5564 Nominal/Abs.thy --- a/Nominal/Abs.thy Wed Apr 14 20:21:11 2010 +0200 +++ b/Nominal/Abs.thy Wed Apr 14 22:23:52 2010 +0200 @@ -762,7 +762,7 @@ by (simp_all add: fresh_plus_perm) -lemma alpha_gen_eqvt[eqvt]: +lemma alpha_gen_eqvt(*[eqvt]*): shows "(bs, x) \gen R f q (cs, y) \ (p \ bs, p \ x) \gen (p \ R) (p \ f) (p \ q) (p \ cs, p \ y)" and "(bs, x) \res R f q (cs, y) \ (p \ bs, p \ x) \res (p \ R) (p \ f) (p \ q) (p \ cs, p \ y)" and "(ds, x) \lst R f q (es, y) \ (p \ ds, p \ x) \lst (p \ R) (p \ f) (p \ q) (p \ es, p \ y)"