src/HOL/IMP/Abs_Int3.thy
changeset 51924 e398ab28eaa7
parent 51914 df962fe09a37
child 51953 ae755fd6c883
--- a/src/HOL/IMP/Abs_Int3.thy	Thu May 09 02:42:51 2013 +0200
+++ b/src/HOL/IMP/Abs_Int3.thy	Thu May 09 03:58:28 2013 +0200
@@ -523,7 +523,7 @@
 lift_definition m_ivl :: "ivl \<Rightarrow> nat" is m_rep
 by(auto simp: m_rep_def eq_ivl_iff)
 
-lemma m_ivl_nice: "m_ivl[l\<dots>h] = (if [l\<dots>h] = \<bottom> then 3 else
+lemma m_ivl_nice: "m_ivl[l,h] = (if [l,h] = \<bottom> then 3 else
    (if l = Minf then 0 else 1) + (if h = Pinf then 0 else 1))"
 unfolding bot_ivl_def
 by transfer (auto simp: m_rep_def eq_ivl_empty split: extended.split)