src/HOL/Real/ContNotDenum.thy
changeset 19765 dfe940911617
parent 19023 5652a536b7e8
child 20635 e95db20977c5
--- 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 \<Rightarrow> real \<Rightarrow> real set"
-  "closed_int x y \<equiv> {z. x \<le> z \<and> z \<le> y}"
+definition
+  closed_int :: "real \<Rightarrow> real \<Rightarrow> real set"
+  "closed_int x y = {z. x \<le> z \<and> z \<le> y}"
 
 subsection {* Properties *}
 
@@ -48,9 +49,9 @@
   {
     fix x::real
     assume "x \<in> closed_int x1 y1"
-    hence "x \<ge> x1 \<and> x \<le> y1" by (unfold closed_int_def, simp)
+    hence "x \<ge> x1 \<and> x \<le> y1" by (simp add: closed_int_def)
     with xy have "x \<ge> x0 \<and> x \<le> y0" by auto
-    hence "x \<in> closed_int x0 y0" by (unfold closed_int_def, simp)
+    hence "x \<in> 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