src/HOL/Real/ContNotDenum.thy
changeset 28562 4e74209f113e
parent 27435 b3f8e9bdf9a7
equal deleted inserted replaced
28561:056255ade52a 28562:4e74209f113e
   401        e = closed_int e1 e2 \<and>
   401        e = closed_int e1 e2 \<and>
   402        e \<subseteq> (newInt n f) \<and>
   402        e \<subseteq> (newInt n f) \<and>
   403        (f (Suc n)) \<notin> e)
   403        (f (Suc n)) \<notin> e)
   404       )"
   404       )"
   405 
   405 
   406 declare newInt.simps [code func del]
   406 declare newInt.simps [code del]
   407 
   407 
   408 subsubsection {* Properties *}
   408 subsubsection {* Properties *}
   409 
   409 
   410 text {* We now show that every application of newInt returns an
   410 text {* We now show that every application of newInt returns an
   411 appropriate interval. *}
   411 appropriate interval. *}