src/HOL/Real/RComplete.thy
changeset 20217 25b068a99d2b
parent 19850 29c125556d86
child 21210 c17fd2df4e9e
--- a/src/HOL/Real/RComplete.thy	Wed Jul 26 13:31:07 2006 +0200
+++ b/src/HOL/Real/RComplete.thy	Wed Jul 26 19:23:04 2006 +0200
@@ -1066,10 +1066,7 @@
   apply (subgoal_tac "real a = real (int a)")
   apply (erule ssubst)
   apply simp
-  apply (subst nat_diff_distrib)
   apply simp
-  apply (rule le_floor)
-  apply simp_all
 done
 
 lemma natceiling_zero [simp]: "natceiling 0 = 0"
@@ -1206,13 +1203,7 @@
   apply (subgoal_tac "real a = real (int a)")
   apply (erule ssubst)
   apply simp
-  apply (subst nat_diff_distrib)
   apply simp
-  apply (rule order_trans)
-  prefer 2
-  apply (rule ceiling_mono2)
-  apply assumption
-  apply simp_all
 done
 
 lemma natfloor_div_nat: "1 <= x ==> 0 < y ==>