src/HOL/Multivariate_Analysis/Integration.thy
changeset 56332 289dd9166d04
parent 56218 1c3f1f2431f9
child 56371 fb9ae0727548
equal deleted inserted replaced
56331:bea2196627cb 56332:289dd9166d04
  8865         done
  8865         done
  8866     qed
  8866     qed
  8867   qed
  8867   qed
  8868   then show ?thesis
  8868   then show ?thesis
  8869     using `x \<in> s` `f c = y` `c \<in> s` by auto
  8869     using `x \<in> s` `f c = y` `c \<in> s` by auto
       
  8870 qed
       
  8871 
       
  8872 lemma has_derivative_zero_connected_constant:
       
  8873   fixes f :: "'a::euclidean_space \<Rightarrow> 'b::banach"
       
  8874   assumes "connected s"
       
  8875       and "open s"
       
  8876       and "finite k"
       
  8877       and "continuous_on s f"
       
  8878       and "\<forall>x\<in>(s - k). (f has_derivative (\<lambda>h. 0)) (at x within s)"
       
  8879     obtains c where "\<And>x. x \<in> s \<Longrightarrow> f(x) = c"
       
  8880 proof (cases "s = {}")
       
  8881   case True
       
  8882   then show ?thesis
       
  8883 by (metis empty_iff that)
       
  8884 next
       
  8885   case False
       
  8886   then obtain c where "c \<in> s"
       
  8887     by (metis equals0I)
       
  8888   then show ?thesis
       
  8889     by (metis has_derivative_zero_unique_strong_connected assms that)
  8870 qed
  8890 qed
  8871 
  8891 
  8872 
  8892 
  8873 subsection {* Integrating characteristic function of an interval *}
  8893 subsection {* Integrating characteristic function of an interval *}
  8874 
  8894