src/HOL/Hyperreal/Integration.thy
changeset 17318 bc1c75855f3d
parent 16924 04246269386e
child 19279 48b527d0331b
equal deleted inserted replaced
17317:3f12de2e2e6e 17318:bc1c75855f3d
   320 apply auto
   320 apply auto
   321 apply (subgoal_tac "\<bar>(rsum (D,p) f - k2) - (rsum (D,p) f - k1)\<bar> < \<bar>k1 - k2\<bar>")
   321 apply (subgoal_tac "\<bar>(rsum (D,p) f - k2) - (rsum (D,p) f - k1)\<bar> < \<bar>k1 - k2\<bar>")
   322 apply arith
   322 apply arith
   323 apply (drule add_strict_mono, assumption)
   323 apply (drule add_strict_mono, assumption)
   324 apply (auto simp only: left_distrib [symmetric] mult_2_right [symmetric] 
   324 apply (auto simp only: left_distrib [symmetric] mult_2_right [symmetric] 
   325                 mult_less_cancel_right, arith)
   325                 mult_less_cancel_right)
       
   326 apply arith
   326 done
   327 done
   327 
   328 
   328 lemma Integral_zero [simp]: "Integral(a,a) f 0"
   329 lemma Integral_zero [simp]: "Integral(a,a) f 0"
   329 apply (auto simp add: Integral_def)
   330 apply (auto simp add: Integral_def)
   330 apply (rule_tac x = "%x. 1" in exI)
   331 apply (rule_tac x = "%x. 1" in exI)