diff -r c7db2ccba18a -r 3a801bbd2687 Correctness.thy --- a/Correctness.thy Wed Feb 03 12:04:03 2016 +0800 +++ b/Correctness.thy Wed Feb 03 21:05:15 2016 +0800 @@ -580,6 +580,7 @@ -- {* All results derived so far hold for both @{term s} and @{term "t@s"}: *} interpret vat_t: extend_highest_gen s th prio tm t using Cons by simp interpret vat_e: extend_highest_gen s th prio tm "(e # t)" using Cons by simp + interpret vat_es: valid_trace_e "t@s" e using Cons(1,2) by (unfold_locales, auto) show ?case proof - -- {* It can be proved that @{term cntP}-value of @{term th'} does not change @@ -591,8 +592,8 @@ -- {* Then the actor of @{term e} must be @{term th'} and @{term e} must be a @{term P}-event: *} hence "isP e" "actor e = th'" by (auto simp:cntP_diff_inv) - with vat_t.actor_inv[OF Cons(2)] - -- {* According to @{thm actor_inv}, @{term th'} must be running at + with vat_es.actor_inv + -- {* According to @{thm vat_es.actor_inv}, @{term th'} must be running at the moment @{term "t@s"}: *} have "th' \ runing (t@s)" by (cases e, auto) -- {* However, an application of @{thm eq_pv_blocked} to induction hypothesis @@ -609,7 +610,7 @@ proof(rule ccontr) -- {* Proof by contradiction. *} assume otherwise: "cntV ((e # t) @ s) th' \ cntV (t @ s) th'" hence "isV e" "actor e = th'" by (auto simp:cntV_diff_inv) - with vat_t.actor_inv[OF Cons(2)] + with vat_es.actor_inv have "th' \ runing (t@s)" by (cases e, auto) moreover have "th' \ runing (t@s)" using vat_t.eq_pv_blocked[OF neq_th' Cons(5)] .