re-arranged class dense_linear_order
authorhaftmann
Mon, 11 Aug 2008 14:50:02 +0200
changeset 27825 12254665fc41
parent 27824 97d2a3797ce0
child 27826 4e50590ea9bc
re-arranged class dense_linear_order
src/HOL/Library/Dense_Linear_Order.thy
src/HOL/Real/PReal.thy
--- a/src/HOL/Library/Dense_Linear_Order.thy	Mon Aug 11 14:50:00 2008 +0200
+++ b/src/HOL/Library/Dense_Linear_Order.thy	Mon Aug 11 14:50:02 2008 +0200
@@ -214,6 +214,10 @@
 context dense_linear_order
 begin
 
+lemma interval_empty_iff:
+  "{y. x < y \<and> y < z} = {} \<longleftrightarrow> \<not> x < z"
+  by (auto dest: dense)
+
 lemma dlo_qe_bnds: 
   assumes ne: "L \<noteq> {}" and neU: "U \<noteq> {}" and fL: "finite L" and fU: "finite U"
   shows "(\<exists>x. (\<forall>y \<in> L. y < x) \<and> (\<forall>y \<in> U. x < y)) \<equiv> (\<forall> l \<in> L. \<forall>u \<in> U. l < u)"
--- a/src/HOL/Real/PReal.thy	Mon Aug 11 14:50:00 2008 +0200
+++ b/src/HOL/Real/PReal.thy	Mon Aug 11 14:50:02 2008 +0200
@@ -10,7 +10,7 @@
 header {* Positive real numbers *}
 
 theory PReal
-imports Rational
+imports Rational Dense_Linear_Order
 begin
 
 text{*Could be generalized and moved to @{text Ring_and_Field}*}