src/HOL/RealVector.thy
changeset 31567 0fb78b3a9145
parent 31565 da5a5589418e
child 31586 d4707b99e631
--- a/src/HOL/RealVector.thy	Thu Jun 11 12:05:41 2009 -0700
+++ b/src/HOL/RealVector.thy	Thu Jun 11 15:33:13 2009 -0700
@@ -828,6 +828,21 @@
   thus "open {a<..<b}" by (simp add: open_Int)
 qed
 
+lemma closed_real_atMost [simp]: 
+  fixes a :: real shows "closed {..a}"
+unfolding closed_open by simp
+
+lemma closed_real_atLeast [simp]:
+  fixes a :: real shows "closed {a..}"
+unfolding closed_open by simp
+
+lemma closed_real_atLeastAtMost [simp]:
+  fixes a b :: real shows "closed {a..b}"
+proof -
+  have "{a..b} = {a..} \<inter> {..b}" by auto
+  thus "closed {a..b}" by (simp add: closed_Int)
+qed
+
 
 subsection {* Extra type constraints *}