cleaned up
authorhaftmann
Thu, 10 May 2007 22:11:37 +0200
changeset 22929 e6b6f8dd03e9
parent 22928 1feef3b54ce1
child 22930 f99617e7103f
cleaned up
src/HOL/Real/Ferrante_Rackoff.thy
--- a/src/HOL/Real/Ferrante_Rackoff.thy	Thu May 10 22:11:36 2007 +0200
+++ b/src/HOL/Real/Ferrante_Rackoff.thy	Thu May 10 22:11:37 2007 +0200
@@ -140,9 +140,6 @@
   \<longrightarrow> (\<forall> y. l < y \<and> y < u \<longrightarrow> (P1 y \<or> P2 y))"
   by blast
 
-declare Max_le_iff [simp]
-declare Max_le_iff [simp]
-
 lemma finite_set_intervals:
   assumes px: "P (x::real)" and lx: "l \<le> x" and xu: "x \<le> u" and linS: "l\<in> S" 
   and uinS: "u \<in> S" and fS:"finite S" and lS: "\<forall> x\<in> S. l \<le> x" and Su: "\<forall> x\<in> S. x \<le> u"