scilib documentation

LeanChemicalTheories / math.antideriv

theorem fun_split (f g : ) :
(λ (x : ), f x + g x) = (λ (x : ), f x) + λ (x : ), g x
theorem antideriv_const (f : ) (k : ) (hf : (x : ), has_deriv_at f k x) :
f = λ (x : ), k * x + f 0
theorem antideriv_pow (f : ) (hf : (x : ) (n : ), has_deriv_at f (x ^ n) x) (n : ) :
f = λ (x : ), x ^ (n + 1) / (n + 1) + f 0
theorem antideriv_zpow (f : ) (hf : (x : ), x 0 (z : ), has_deriv_at f (x ^ z) x) (z : ) :
z + 1 0 (f = λ (x : ), x ^ (z + 1) / (z + 1) + f 0)
theorem antideriv_first_order_poly {k j : } (f : ) (hf : (x : ), has_deriv_at f (j * x + k) x) :
f = λ (x : ), j * x ^ 2 / 2 + k * x + f 0
theorem constant_of_has_deriv_right_zero' {E : Type u_1} [normed_add_comm_group E] [normed_space E] {f : E} {a b : } (hderiv : (x : ), x set.Icc a b has_deriv_at f 0 x) (h : a b) :
f b = f a
theorem antideriv {E : Type u_2} {𝕜 : Type u_3} [is_R_or_C 𝕜] [normed_add_comm_group E] [normed_space 𝕜 E] {f F G : 𝕜 E} (hf : (t : 𝕜), has_deriv_at F (f t) t) (hg : (t : 𝕜), has_deriv_at G (f t) t) (hg' : G 0 = 0) :
F = λ (t : 𝕜), G t + F 0
theorem has_deriv_at_linear_no_pow {𝕜 : Type u_3} [is_R_or_C 𝕜] (x : 𝕜) :
has_deriv_at (λ (y : 𝕜), y) 1 x
theorem antideriv_const' {E : Type u_2} {𝕜 : Type u_3} [is_R_or_C 𝕜] [normed_add_comm_group E] [normed_space 𝕜 E] (f : 𝕜 E) {k : E} (hf : (x : 𝕜), has_deriv_at f k x) :
f = λ (x : 𝕜), x k + f 0
theorem antideriv_first_order_poly' {E : Type u_2} {𝕜 : Type u_3} [is_R_or_C 𝕜] [normed_add_comm_group E] [normed_space 𝕜 E] {k j : E} (f : 𝕜 E) (hf : (x : 𝕜), has_deriv_at f (x j + k) x) :
f = λ (x : 𝕜), (x ^ 2 / 2) j + x k + f 0

Analytical ODE solutions #