Smoothness of Real.sqrt #
In this file we prove that Real.sqrt is infinitely smooth at all points x ≠ 0 and provide some
dot-notation lemmas.
Tags #
sqrt, differentiable
Local homeomorph between (0, +∞) and (0, +∞) with toFun = (· ^ 2) and
invFun = Real.sqrt.
Equations
- One or more equations did not get rendered due to their size.
Instances For
theorem
HasStrictDerivAt.sqrt
{f : ℝ → ℝ}
{f' : ℝ}
{x : ℝ}
(hf : HasStrictDerivAt f f' x)
(hx : f x ≠ 0)
 :
theorem
derivWithin_sqrt
{f : ℝ → ℝ}
{s : Set ℝ}
{x : ℝ}
(hf : DifferentiableWithinAt ℝ f s x)
(hx : f x ≠ 0)
(hxs : UniqueDiffWithinAt ℝ s x)
 :
derivWithin (fun (x : ℝ) => √(f x)) s x = derivWithin f s x / (2 * √(f x))
theorem
HasFDerivAt.sqrt
{E : Type u_1}
[NormedAddCommGroup E]
[NormedSpace ℝ E]
{f : E → ℝ}
{x : E}
{f' : E →L[ℝ] ℝ}
(hf : HasFDerivAt f f' x)
(hx : f x ≠ 0)
 :
theorem
HasStrictFDerivAt.sqrt
{E : Type u_1}
[NormedAddCommGroup E]
[NormedSpace ℝ E]
{f : E → ℝ}
{x : E}
{f' : E →L[ℝ] ℝ}
(hf : HasStrictFDerivAt f f' x)
(hx : f x ≠ 0)
 :
theorem
HasFDerivWithinAt.sqrt
{E : Type u_1}
[NormedAddCommGroup E]
[NormedSpace ℝ E]
{f : E → ℝ}
{s : Set E}
{x : E}
{f' : E →L[ℝ] ℝ}
(hf : HasFDerivWithinAt f f' s x)
(hx : f x ≠ 0)
 :
theorem
DifferentiableWithinAt.sqrt
{E : Type u_1}
[NormedAddCommGroup E]
[NormedSpace ℝ E]
{f : E → ℝ}
{s : Set E}
{x : E}
(hf : DifferentiableWithinAt ℝ f s x)
(hx : f x ≠ 0)
 :
DifferentiableWithinAt ℝ (fun (y : E) => √(f y)) s x
theorem
DifferentiableAt.sqrt
{E : Type u_1}
[NormedAddCommGroup E]
[NormedSpace ℝ E]
{f : E → ℝ}
{x : E}
(hf : DifferentiableAt ℝ f x)
(hx : f x ≠ 0)
 :
DifferentiableAt ℝ (fun (y : E) => √(f y)) x
theorem
DifferentiableOn.sqrt
{E : Type u_1}
[NormedAddCommGroup E]
[NormedSpace ℝ E]
{f : E → ℝ}
{s : Set E}
(hf : DifferentiableOn ℝ f s)
(hs : ∀ x ∈ s, f x ≠ 0)
 :
DifferentiableOn ℝ (fun (y : E) => √(f y)) s
theorem
Differentiable.sqrt
{E : Type u_1}
[NormedAddCommGroup E]
[NormedSpace ℝ E]
{f : E → ℝ}
(hf : Differentiable ℝ f)
(hs : ∀ (x : E), f x ≠ 0)
 :
Differentiable ℝ fun (y : E) => √(f y)
theorem
fderivWithin_sqrt
{E : Type u_1}
[NormedAddCommGroup E]
[NormedSpace ℝ E]
{f : E → ℝ}
{s : Set E}
{x : E}
(hf : DifferentiableWithinAt ℝ f s x)
(hx : f x ≠ 0)
(hxs : UniqueDiffWithinAt ℝ s x)
 :
fderivWithin ℝ (fun (x : E) => √(f x)) s x = (1 / (2 * √(f x))) • fderivWithin ℝ f s x
@[simp]
theorem
fderiv_sqrt
{E : Type u_1}
[NormedAddCommGroup E]
[NormedSpace ℝ E]
{f : E → ℝ}
{x : E}
(hf : DifferentiableAt ℝ f x)
(hx : f x ≠ 0)
 :
theorem
ContDiffAt.sqrt
{E : Type u_1}
[NormedAddCommGroup E]
[NormedSpace ℝ E]
{f : E → ℝ}
{n : ℕ∞}
{x : E}
(hf : ContDiffAt ℝ n f x)
(hx : f x ≠ 0)
 :
ContDiffAt ℝ n (fun (y : E) => √(f y)) x
theorem
ContDiffWithinAt.sqrt
{E : Type u_1}
[NormedAddCommGroup E]
[NormedSpace ℝ E]
{f : E → ℝ}
{n : ℕ∞}
{s : Set E}
{x : E}
(hf : ContDiffWithinAt ℝ n f s x)
(hx : f x ≠ 0)
 :
ContDiffWithinAt ℝ n (fun (y : E) => √(f y)) s x
theorem
ContDiffOn.sqrt
{E : Type u_1}
[NormedAddCommGroup E]
[NormedSpace ℝ E]
{f : E → ℝ}
{n : ℕ∞}
{s : Set E}
(hf : ContDiffOn ℝ n f s)
(hs : ∀ x ∈ s, f x ≠ 0)
 :
ContDiffOn ℝ n (fun (y : E) => √(f y)) s
theorem
ContDiff.sqrt
{E : Type u_1}
[NormedAddCommGroup E]
[NormedSpace ℝ E]
{f : E → ℝ}
{n : ℕ∞}
(hf : ContDiff ℝ n f)
(h : ∀ (x : E), f x ≠ 0)
 :