simp del: empty_Collect_eq;
authorwenzelm
Sat, 17 Dec 2005 01:58:41 +0100
changeset 18429 42ee9f24f63a
parent 18428 4059413acbc1
child 18430 46c18c0b52c1
simp del: empty_Collect_eq;
src/HOL/Real/PReal.thy
--- a/src/HOL/Real/PReal.thy	Sat Dec 17 01:00:40 2005 +0100
+++ b/src/HOL/Real/PReal.thy	Sat Dec 17 01:58:41 2005 +0100
@@ -139,7 +139,7 @@
 subsection{*@{term preal_of_prat}: the Injection from prat to preal*}
 
 lemma rat_less_set_mem_preal: "0 < y ==> {u::rat. 0 < u & u < y} \<in> preal"
-apply (auto simp add: preal_def cut_def intro: order_less_trans)
+apply (auto simp del: empty_Collect_eq simp add: preal_def cut_def intro: order_less_trans)
 apply (force simp only: eq_commute [of "{}"] interval_empty_iff)
 apply (blast dest: dense intro: order_less_trans)
 done