--- a/Nominal/Ex/CPS/CPS2_DanvyNielsen.thy Thu Mar 13 09:30:26 2014 +0000
+++ b/Nominal/Ex/CPS/CPS2_DanvyNielsen.thy Mon Mar 24 15:31:17 2014 +0000
@@ -48,7 +48,6 @@
apply (rule_tac y="a" and c="b" in cpsctxt.strong_exhaust)
using [[simproc del: alpha_lst]]
apply (auto simp add: fresh_star_def)
- apply blast+
apply (erule Abs_lst1_fcb)
apply (simp_all add: Abs_fresh_iff)
apply (erule fresh_eqvt_at)
@@ -82,7 +81,6 @@
apply (rule_tac y="a" in lt.exhaust)
using [[simproc del: alpha_lst]]
apply auto
- apply blast
apply (rule_tac x="lt" and ?'a="name" in obtain_fresh)
apply (simp add: Abs1_eq_iff)
apply blast+