File tree Expand file tree Collapse file tree 1 file changed +6
-5
lines changed
Mathlib/Analysis/SpecialFunctions Expand file tree Collapse file tree 1 file changed +6
-5
lines changed Original file line number Diff line number Diff line change @@ -145,12 +145,11 @@ end ComplexContinuousExpComp
145145
146146namespace 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
155154lemma 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
181180theorem ContinuousWithinAt.rexp (h : ContinuousWithinAt f s x) :
182181 ContinuousWithinAt (fun y ↦ exp (f y)) s x :=
183182 h.rexp
183+
184184@[fun_prop]
185185nonrec
186186theorem 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]
351352theorem isOpenEmbedding_exp : IsOpenEmbedding exp :=
352353 isOpen_Ioi.isOpenEmbedding_subtypeVal.comp expOrderIso.toHomeomorph.isOpenEmbedding
353354
You can’t perform that action at this time.
0 commit comments