src/HOL/IMP/Abs_Int3.thy
changeset 51786 61ed47755088
parent 51785 9685a5b1f7ce
child 51791 c4db685eaed0
--- a/src/HOL/IMP/Abs_Int3.thy	Fri Apr 26 09:41:45 2013 +0200
+++ b/src/HOL/IMP/Abs_Int3.thy	Fri Apr 26 09:53:11 2013 +0200
@@ -398,7 +398,7 @@
 lemma m_c_widen:
   "strip C1 = strip C2  \<Longrightarrow> top_on_acom C1 (-vars C1) \<Longrightarrow> top_on_acom C2 (-vars C2)
    \<Longrightarrow> \<not> C2 \<le> C1 \<Longrightarrow> m_c (C1 \<nabla> C2) < m_c C1"
-apply(auto simp: m_c_def widen_acom_def)
+apply(auto simp: m_c_def widen_acom_def listsum_setsum_nth atLeast0LessThan)
 apply(subgoal_tac "length(annos C2) = length(annos C1)")
  prefer 2 apply (simp add: size_annos_same2)
 apply (auto)