Skip to content

Commit

Permalink
chore(analysis/special_functions/pow): put lemmas about derivatives i…
Browse files Browse the repository at this point in the history
…nto a new file (#10153)

In order to keep results about continuity of the power function in the original file, we prove some continuity results directly (these were previously proved using derivatives).



Co-authored-by: RemyDegenne <remydegenne@gmail.com>
  • Loading branch information
RemyDegenne and RemyDegenne committed Nov 12, 2021
1 parent 75207e9 commit c45e70a
Show file tree
Hide file tree
Showing 6 changed files with 664 additions and 505 deletions.
1 change: 1 addition & 0 deletions archive/100-theorems-list/9_area_of_a_circle.lean
Expand Up @@ -5,6 +5,7 @@ Authors: James Arthur, Benjamin Davidson, Andrew Souther
-/
import measure_theory.integral.interval_integral
import analysis.special_functions.sqrt
import analysis.special_functions.trigonometric.inverse_deriv

/-!
# Freek № 9: The Area of a Circle
Expand Down
1 change: 1 addition & 0 deletions src/analysis/complex/polynomial.lean
Expand Up @@ -5,6 +5,7 @@ Authors: Chris Hughes
-/
import analysis.special_functions.pow
import field_theory.is_alg_closed.basic
import topology.algebra.polynomial

/-!
# The fundamental theorem of algebra
Expand Down
2 changes: 1 addition & 1 deletion src/analysis/convex/specific_functions.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yury Kudryashov, Sébastien Gouëzel
-/
import analysis.calculus.mean_value
import analysis.special_functions.pow
import analysis.special_functions.pow_deriv

/-!
# Collection of convex functions
Expand Down

0 comments on commit c45e70a

Please sign in to comment.