diff -r e08e3c29dbc0 -r 2205b572bc9b Nominal/Abs.thy --- a/Nominal/Abs.thy Tue May 11 14:58:46 2010 +0100 +++ b/Nominal/Abs.thy Tue May 11 17:16:57 2010 +0200 @@ -760,7 +760,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)"