Skip to content

Commit 728f668

Browse files
committed
chore(Analysis/SpecialFunctions/Exp): use fun_prop more (#31304)
Golf a few proofs with it, and tag a few more lemmas. Noticed in passing, why not improve the tagging here?
1 parent c03aec9 commit 728f668

File tree

1 file changed

+6
-5
lines changed
  • Mathlib/Analysis/SpecialFunctions

1 file changed

+6
-5
lines changed

Mathlib/Analysis/SpecialFunctions/Exp.lean

Lines changed: 6 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -145,12 +145,11 @@ end ComplexContinuousExpComp
145145

146146
namespace Real
147147

148-
@[continuity]
149-
theorem continuous_exp : Continuous exp :=
150-
Complex.continuous_re.comp Complex.continuous_ofReal.cexp
148+
@[continuity, fun_prop]
149+
theorem continuous_exp : Continuous exp := by
150+
unfold Real.exp; fun_prop
151151

152-
theorem continuousOn_exp {s : Set ℝ} : ContinuousOn exp s :=
153-
continuous_exp.continuousOn
152+
theorem continuousOn_exp {s : Set ℝ} : ContinuousOn exp s := by fun_prop
154153

155154
lemma exp_sub_sum_range_isBigO_pow (n : ℕ) :
156155
(fun x ↦ exp x - ∑ i ∈ Finset.range n, x ^ i / i !) =O[𝓝 0] (· ^ n) := by
@@ -181,6 +180,7 @@ nonrec
181180
theorem ContinuousWithinAt.rexp (h : ContinuousWithinAt f s x) :
182181
ContinuousWithinAt (fun y ↦ exp (f y)) s x :=
183182
h.rexp
183+
184184
@[fun_prop]
185185
nonrec
186186
theorem ContinuousAt.rexp (h : ContinuousAt f x) : ContinuousAt (fun y ↦ exp (f y)) x :=
@@ -348,6 +348,7 @@ theorem tendsto_exp_comp_nhds_zero {f : α → ℝ} :
348348
Tendsto (fun x => exp (f x)) l (𝓝 0) ↔ Tendsto f l atBot := by
349349
simp_rw [← comp_apply (f := exp), ← tendsto_comap_iff, comap_exp_nhds_zero]
350350

351+
@[fun_prop]
351352
theorem isOpenEmbedding_exp : IsOpenEmbedding exp :=
352353
isOpen_Ioi.isOpenEmbedding_subtypeVal.comp expOrderIso.toHomeomorph.isOpenEmbedding
353354

0 commit comments

Comments
 (0)