diff -r 5a0d1075911c -r a1de627d417a src/HOL/Analysis/Complex_Transcendental.thy --- a/src/HOL/Analysis/Complex_Transcendental.thy Mon Apr 07 12:36:56 2025 +0200 +++ b/src/HOL/Analysis/Complex_Transcendental.thy Tue Apr 08 19:06:00 2025 +0100 @@ -2919,6 +2919,16 @@ qed (use z in auto) qed +lemma has_field_derivative_csqrt' [derivative_intros]: + assumes "(f has_field_derivative f') (at x within A)" "f x \ \\<^sub>\\<^sub>0" + shows "((\x. csqrt (f x)) has_field_derivative (f' / (2 * csqrt (f x)))) (at x within A)" +proof - + have "((csqrt \ f) has_field_derivative (inverse (2 * csqrt (f x)) * f')) (at x within A)" + using has_field_derivative_csqrt assms(1) by (rule DERIV_chain) fact + thus ?thesis + by (simp add: o_def field_simps) +qed + lemma field_differentiable_at_csqrt: "z \ \\<^sub>\\<^sub>0 \ csqrt field_differentiable at z" using field_differentiable_def has_field_derivative_csqrt by blast