diff -r de51a86fc903 -r cc97b347b301 src/HOL/IMP/Abs_Int1.thy --- a/src/HOL/IMP/Abs_Int1.thy Fri Jul 04 20:07:08 2014 +0200 +++ b/src/HOL/IMP/Abs_Int1.thy Fri Jul 04 20:18:47 2014 +0200 @@ -109,7 +109,7 @@ "m_s S X = (\ x \ X. m(fun S x))" lemma m_s_h: "finite X \ m_s S X \ h * card X" -by(simp add: m_s_def) (metis nat_mult_commute of_nat_id setsum_bounded[OF h]) +by(simp add: m_s_def) (metis mult.commute of_nat_id setsum_bounded[OF h]) definition m_o :: "'av st option \ vname set \ nat" ("m\<^sub>o") where "m_o opt X = (case opt of None \ h * card X + 1 | Some S \ m_s S X)"