diff -r eae86cba8b89 -r 550ab0f68960 Correctness.thy --- a/Correctness.thy Mon Mar 06 13:11:16 2017 +0000 +++ b/Correctness.thy Thu Mar 16 13:20:46 2017 +0000 @@ -1255,6 +1255,30 @@ finally show ?thesis . qed +value "sublists [a,b,cThe]" + +theorem bound_priority_inversion: + "card { s' @ s | s'. s' \ set t \ th \ running (s'@s) } \ + 1 + (length (actions_of blockers t) + length (filter (isCreate) t))" + (is "?L \ ?R") +proof - + let ?Q = "(\ t'. th \ running (t'@s))" + from occs_le[of ?Q t] + have "?L \ (1 + length t) - occs ?Q t" by simp + also have "... \ ?R" + proof - + have "length t - (length (actions_of blockers t) + length (filter (isCreate) t)) + \ occs (\ t'. th \ running (t'@s)) t" (is "?L1 \ ?R1") + proof - + have "?L1 = length (actions_of {th} t)" using actions_split by arith + also have "... \ ?R1" using actions_th_occs by simp + finally show ?thesis . + qed + thus ?thesis by simp + qed + finally show ?thesis . +qed + end text {*