diff -r 4ccb7e6be929 -r 51a80e238b29 src/HOL/MicroJava/BV/EffectMono.thy --- a/src/HOL/MicroJava/BV/EffectMono.thy Wed Feb 07 17:41:11 2007 +0100 +++ b/src/HOL/MicroJava/BV/EffectMono.thy Wed Feb 07 17:44:07 2007 +0100 @@ -10,7 +10,7 @@ lemma PrimT_PrimT: "(G \ xb \ PrimT p) = (xb = PrimT p)" - by (auto elim: widen.elims) + by (auto elim: widen.cases) lemma sup_loc_some [rule_format]: @@ -42,7 +42,7 @@ lemma all_widen_is_sup_loc: "\b. length a = length b \ - (\x\set (zip a b). x \ widen G) = (G \ (map OK a) <=l (map OK b))" + (\(x, y)\set (zip a b). G \ x \ y) = (G \ (map OK a) <=l (map OK b))" (is "\b. length a = length b \ ?Q a b" is "?P a") proof (induct "a") show "?P []" by simp @@ -219,7 +219,7 @@ l: "length apTs = length list" and c: "is_class G cname" and C: "G \ X \ Class cname" and - w: "\x \ set (zip apTs list). x \ widen G" and + w: "\(x, y) \ set (zip apTs list). G \ x \ y" and m: "method (G, cname) (mname, list) = Some (mD', rT', b')" and x: "\C \ set (match_any G pc et). is_class G C" by (simp del: not_None_eq, elim exE conjE) (rule that) @@ -261,7 +261,7 @@ have "G \ map OK apTs' <=l map OK list" . with l' - have w': "\x \ set (zip apTs' list). x \ widen G" + have w': "\(x, y) \ set (zip apTs' list). G \ x \ y" by (simp add: all_widen_is_sup_loc) from Invoke s2 l' w' C' m c x