diff -r 372065f34795 -r dfe940911617 src/HOL/Real/ContNotDenum.thy --- a/src/HOL/Real/ContNotDenum.thy Fri Jun 02 20:12:59 2006 +0200 +++ b/src/HOL/Real/ContNotDenum.thy Fri Jun 02 23:22:29 2006 +0200 @@ -36,8 +36,9 @@ subsection {* Definition *} -constdefs closed_int :: "real \ real \ real set" - "closed_int x y \ {z. x \ z \ z \ y}" +definition + closed_int :: "real \ real \ real set" + "closed_int x y = {z. x \ z \ z \ y}" subsection {* Properties *} @@ -48,9 +49,9 @@ { fix x::real assume "x \ closed_int x1 y1" - hence "x \ x1 \ x \ y1" by (unfold closed_int_def, simp) + hence "x \ x1 \ x \ y1" by (simp add: closed_int_def) with xy have "x \ x0 \ x \ y0" by auto - hence "x \ closed_int x0 y0" by (unfold closed_int_def, simp) + hence "x \ closed_int x0 y0" by (simp add: closed_int_def) } thus ?thesis by auto qed @@ -575,4 +576,4 @@ ultimately show False by blast qed -end \ No newline at end of file +end