diff -r 6d6cb845e841 -r fc0b575a2cf7 src/HOL/MicroJava/BV/Correct.thy --- a/src/HOL/MicroJava/BV/Correct.thy Tue Dec 05 14:08:22 2000 +0100 +++ b/src/HOL/MicroJava/BV/Correct.thy Tue Dec 05 14:08:56 2000 +0100 @@ -38,16 +38,16 @@ "correct_frames G hp phi rT0 sig0 (f#frs) = (let (stk,loc,C,sig,pc) = f in - (\ST LT rT maxl ins. + (\ST LT rT maxs maxl ins. phi C sig ! pc = Some (ST,LT) \ - method (G,C) sig = Some(C,rT,(maxl,ins)) \ + method (G,C) sig = Some(C,rT,(maxs,maxl,ins)) \ (\C' mn pTs k. pc = k+1 \ ins!k = (Invoke C' mn pTs) \ (mn,pTs) = sig0 \ (\apTs D ST' LT'. (phi C sig)!k = Some ((rev apTs) @ (Class D) # ST', LT') \ length apTs = length pTs \ - (\D' rT' maxl' ins'. - method (G,D) sig0 = Some(D',rT',(maxl',ins')) \ + (\D' rT' maxs' maxl' ins'. + method (G,D) sig0 = Some(D',rT',(maxs',maxl',ins')) \ G \ rT0 \ rT') \ correct_frame G hp (tl ST, LT) maxl ins f \ correct_frames G hp phi rT sig frs))))" @@ -63,8 +63,8 @@ | (f#fs) => G\h hp\ \ (let (stk,loc,C,sig,pc) = f in - \rT maxl ins s. - method (G,C) sig = Some(C,rT,(maxl,ins)) \ + \rT maxs maxl ins s. + method (G,C) sig = Some(C,rT,(maxs,maxl,ins)) \ phi C sig ! pc = Some s \ correct_frame G hp s maxl ins f \ correct_frames G hp phi rT sig fs))