src/HOL/Set_Interval.thy
changeset 52729 412c9e0381a1
parent 52380 3cc46b8cca5e
child 53216 ad2e09c30aa8
--- a/src/HOL/Set_Interval.thy	Wed Jul 24 17:15:59 2013 +0200
+++ b/src/HOL/Set_Interval.thy	Thu Jul 25 08:57:16 2013 +0200
@@ -197,8 +197,8 @@
 by (simp add: atLeastAtMost_def)
 
 text {* The above four lemmas could be declared as iffs. Unfortunately this
-breaks many proofs. Since it only helps blast, it is better to leave well
-alone *}
+breaks many proofs. Since it only helps blast, it is better to leave them
+alone. *}
 
 lemma greaterThanLessThan_eq: "{ a <..< b} = { a <..} \<inter> {..< b }"
   by auto
@@ -452,10 +452,10 @@
   shows "{a ..< b} = {c ..< d} \<longleftrightarrow> a = c \<and> b = d"
   using atLeastLessThan_inj assms by auto
 
-lemma (in bot) atLeast_eq_UNIV_iff: "{x..} = UNIV \<longleftrightarrow> x = bot"
+lemma (in order_bot) atLeast_eq_UNIV_iff: "{x..} = UNIV \<longleftrightarrow> x = bot"
 by (auto simp: set_eq_iff intro: le_bot)
 
-lemma (in top) atMost_eq_UNIV_iff: "{..x} = UNIV \<longleftrightarrow> x = top"
+lemma (in order_top) atMost_eq_UNIV_iff: "{..x} = UNIV \<longleftrightarrow> x = top"
 by (auto simp: set_eq_iff intro: top_le)
 
 lemma (in bounded_lattice) atLeastAtMost_eq_UNIV_iff: