author | Christian Urban <urbanc@in.tum.de> |
Sun, 07 Feb 2010 10:20:29 +0100 | |
changeset 1080 | 2f1377bb4e1f |
parent 1079 | c70e7545b738 |
child 1081 | 11895d5e3d49 |
--- a/Quot/Nominal/Nominal2_Supp.thy Sun Feb 07 10:16:21 2010 +0100 +++ b/Quot/Nominal/Nominal2_Supp.thy Sun Feb 07 10:20:29 2010 +0100 @@ -153,7 +153,7 @@ thus "h a = h b" by simp next assume "a \<noteq> b" - hence "atom a \<sharp> b" by (simp add: fresh_at) + hence "atom a \<sharp> b" by (simp add: fresh_at_base) with a3 have "atom a \<sharp> h b" by (rule fresh_apply) with a2 have d1: "(atom b \<rightleftharpoons> atom a) \<bullet> (h b) = (h b)" by (rule swap_fresh_fresh)