src/HOL/SetInterval.thy
changeset 39302 d7728f65b353
parent 39198 f967a16dfcdd
child 40703 d1fc454d6735
--- a/src/HOL/SetInterval.thy	Mon Sep 13 08:43:48 2010 +0200
+++ b/src/HOL/SetInterval.thy	Mon Sep 13 11:13:15 2010 +0200
@@ -241,7 +241,7 @@
 lemma atLeastatMost_psubset_iff:
   "{a..b} < {c..d} \<longleftrightarrow>
    ((~ a <= b) | c <= a & b <= d & (c < a | b < d))  &  c <= d"
-by(simp add: psubset_eq set_ext_iff less_le_not_le)(blast intro: order_trans)
+by(simp add: psubset_eq set_eq_iff less_le_not_le)(blast intro: order_trans)
 
 lemma atLeastAtMost_singleton_iff[simp]:
   "{a .. b} = {c} \<longleftrightarrow> a = b \<and> b = c"