--- a/Init_prop.thy Tue May 21 08:01:33 2013 +0800
+++ b/Init_prop.thy Tue May 21 10:19:51 2013 +0800
@@ -709,10 +709,11 @@
apply (simp only:cpfd2sfds_def init_cfds2sfds_def)
apply (rule set_eqI, rule iffI)
apply (drule CollectD, rule CollectI, (erule exE)+)
-apply (rule_tac x = fd in exI, rule_tac x = sfd in exI, rule_tac x = f in exI) defer
+apply (rule_tac x = fd in exI, rule_tac x = f in exI) defer
apply (drule CollectD, rule CollectI, (erule exE)+)
-apply (rule_tac x = fd in exI, rule_tac x = sfd in exI, rule_tac x = f in exI)
-using cfd2sfd_nil_prop by auto
+apply (rule_tac x = fd in exI, rule_tac x = f in exI)
+using cfd2sfd_nil_prop
+by auto
lemma ch2sshm_nil_prop:
"h \<in> init_shms \<Longrightarrow> ch2sshm [] h = init_ch2sshm h"