diff -r 751d1349329b -r 56b849d348ae Nominal/Ex/ExLetRec.thy --- a/Nominal/Ex/ExLetRec.thy Mon May 10 15:45:04 2010 +0200 +++ b/Nominal/Ex/ExLetRec.thy Mon May 10 15:54:16 2010 +0200 @@ -7,7 +7,6 @@ atom_decl name -ML {* val _ = cheat_alpha_eqvt := true *} ML {* val _ = cheat_equivp := true *} nominal_datatype trm = @@ -83,12 +82,6 @@ apply (simp add: atom_eqvt fresh_star_def) done -(* -declare permute_trm_raw_permute_lts_raw.simps[eqvt] -declare alpha_gen_eqvt[eqvt] -equivariance alpha_trm_raw -*) - end