new lemmas
authorhuffman
Thu, 11 Jun 2009 15:33:13 -0700
changeset 31567 0fb78b3a9145
parent 31566 eff95000aae7
child 31568 963caf6fa234
new lemmas
src/HOL/RealVector.thy
--- 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 *}