src/HOL/IMP/Abs_Int1.thy
changeset 57512 cc97b347b301
parent 55010 203b4f5482c3
child 60974 6a6f15d8fbc4
--- 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 = (\<Sum> x \<in> X. m(fun S x))"
 
 lemma m_s_h: "finite X \<Longrightarrow> m_s S X \<le> 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 \<Rightarrow> vname set \<Rightarrow> nat" ("m\<^sub>o") where
 "m_o opt X = (case opt of None \<Rightarrow> h * card X + 1 | Some S \<Rightarrow> m_s S X)"