diff -r 886655a150f6 -r d1b97708d5eb src/HOL/MicroJava/BV/LBVComplete.thy --- a/src/HOL/MicroJava/BV/LBVComplete.thy Thu Jun 21 20:48:48 2007 +0200 +++ b/src/HOL/MicroJava/BV/LBVComplete.thy Thu Jun 21 22:10:16 2007 +0200 @@ -346,7 +346,7 @@ with s_phi pc phi_pc have wt_s_phi: "wtc c pc s <=_r wtc c pc (\!pc)" by (rule wtc_mono) with wt_phi have wt_s: "wtc c pc s \ \" by simp moreover - assume s: "s \ \" + assume s': "s \ \" ultimately have "ls = [] \ ?wtl (i#ls) pc s \ \" by simp moreover { @@ -357,23 +357,23 @@ moreover from cert suc_pc have "c!pc \ A" "c!(pc+1) \ A" by (auto simp add: cert_ok_def) - with pres have "wtc c pc s \ A" by (rule wtc_pres) + from pres this s pc have "wtc c pc s \ A" by (rule wtc_pres) ultimately have "?wtl ls (Suc pc) (wtc c pc s) \ \" using IH wt_s by blast - with s wt_s have "?wtl (i#ls) pc s \ \" by simp + with s' wt_s have "?wtl (i#ls) pc s \ \" by simp } ultimately show "?wtl (i#ls) pc s \ \" by (cases ls) blast+ qed theorem (in lbvc) wtl_complete: - assumes "wt_step r \ step \" - assumes "s <=_r \!0" and "s \ A" and "s \ \" and "length ins = length phi" + assumes wt: "wt_step r \ step \" + and s: "s <=_r \!0" "s \ A" "s \ \" + and len: "length ins = length phi" shows "wtl ins c 0 s \ \" -proof - - have "0+length ins = length phi" by simp - thus ?thesis by - (rule wt_step_wtl_lemma) +proof - + from len have "0+length ins = length phi" by simp + from wt this s show ?thesis by (rule wt_step_wtl_lemma) qed - end