src/HOL/Multivariate_Analysis/Integration.thy
changeset 35752 c8a8df426666
parent 35751 f7f8d59b60b9
child 35945 fcd02244e63d
equal deleted inserted replaced
35751:f7f8d59b60b9 35752:c8a8df426666
  3906     show "\<exists>B>0. \<forall>a b. ball 0 B \<subseteq> {a..b} \<longrightarrow>
  3906     show "\<exists>B>0. \<forall>a b. ball 0 B \<subseteq> {a..b} \<longrightarrow>
  3907                     norm (integral {a..b} (\<lambda>x. if x \<in> s then f x else 0) - i) < e"
  3907                     norm (integral {a..b} (\<lambda>x. if x \<in> s then f x else 0) - i) < e"
  3908     proof(rule,rule,rule B,safe) case goal1 from B(2)[OF this] guess z .. note z=conjunctD2[OF this]
  3908     proof(rule,rule,rule B,safe) case goal1 from B(2)[OF this] guess z .. note z=conjunctD2[OF this]
  3909       from integral_unique[OF this(1)] show ?case using z(2) by auto qed qed qed 
  3909       from integral_unique[OF this(1)] show ?case using z(2) by auto qed qed qed 
  3910 
  3910 
       
  3911 
       
  3912 
       
  3913 declare [[smt_certificates=""]]
       
  3914 
  3911 end
  3915 end