Skip to content

Commit

Permalink
chore(analysis/special_functions/exp_deriv): downgrade import (#19139)
Browse files Browse the repository at this point in the history
Move lemma `complex.is_open_map_exp` from `special_functions/exp_deriv` to right before its (unique) place of use, in `complex.exp_local_homeomorph` in `special_functions/log_deriv`.  Morally these belong together: being an open map and being a local homeomorphism are closely tied, they are both consequences of the inverse function theorem and the point of both is to set up being able to differentiate complex log as the inverse function of complex exp.

This removes the inverse function theorem from the dependencies of `special_functions/exp_deriv` (a surprisingly widely-imported file).
  • Loading branch information
hrmacbeth committed Jun 2, 2023
1 parent 34ebaff commit 6a5c850
Show file tree
Hide file tree
Showing 2 changed files with 4 additions and 4 deletions.
4 changes: 4 additions & 0 deletions src/analysis/special_functions/complex/log_deriv.lean
Expand Up @@ -3,6 +3,7 @@ Copyright (c) 2018 Chris Hughes. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Chris Hughes, Abhimanyu Pallavi Sudhir, Jean Lo, Calle Sönne, Benjamin Davidson
-/
import analysis.calculus.inverse
import analysis.special_functions.complex.log
import analysis.special_functions.exp_deriv

Expand All @@ -19,6 +20,9 @@ open set filter

open_locale real topology

lemma is_open_map_exp : is_open_map exp :=
open_map_of_strict_deriv has_strict_deriv_at_exp exp_ne_zero

/-- `complex.exp` as a `local_homeomorph` with `source = {z | -π < im z < π}` and
`target = {z | 0 < re z} ∪ {z | im z ≠ 0}`. This definition is used to prove that `complex.log`
is complex differentiable at all points but the negative real semi-axis. -/
Expand Down
4 changes: 0 additions & 4 deletions src/analysis/special_functions/exp_deriv.lean
Expand Up @@ -3,7 +3,6 @@ Copyright (c) 2018 Chris Hughes. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Chris Hughes, Abhimanyu Pallavi Sudhir, Jean Lo, Calle Sönne
-/
import analysis.calculus.inverse
import analysis.complex.real_deriv

/-!
Expand Down Expand Up @@ -67,9 +66,6 @@ lemma has_strict_fderiv_at_exp_real (x : ℂ) :
has_strict_fderiv_at exp (exp x • (1 : ℂ →L[ℝ] ℂ)) x :=
(has_strict_deriv_at_exp x).complex_to_real_fderiv

lemma is_open_map_exp : is_open_map exp :=
open_map_of_strict_deriv has_strict_deriv_at_exp exp_ne_zero

end complex

section
Expand Down

0 comments on commit 6a5c850

Please sign in to comment.