Skip to content

Commit e4e3f2f

Browse files
committed
chore: exp -> NormedSpace.exp (#8436)
Per discussion at [zulip](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Real.2Eexp/near/401485920) Co-authored-by: Scott Morrison <[email protected]>
1 parent 19210bc commit e4e3f2f

File tree

12 files changed

+125
-91
lines changed

12 files changed

+125
-91
lines changed

Mathlib/Analysis/NormedSpace/DualNumber.lean

+1
Original file line numberDiff line numberDiff line change
@@ -19,6 +19,7 @@ These are just restatements of similar statements about `TrivSqZeroExt R M`.
1919
2020
-/
2121

22+
open NormedSpace -- For `exp`.
2223

2324
namespace DualNumber
2425

Mathlib/Analysis/NormedSpace/Exponential.lean

+107-83
Large diffs are not rendered by default.

Mathlib/Analysis/NormedSpace/MatrixExponential.lean

+2
Original file line numberDiff line numberDiff line change
@@ -62,6 +62,8 @@ results for general rings are instead stated about `Ring.inverse`:
6262

6363
open scoped Matrix BigOperators
6464

65+
open NormedSpace -- For `exp`.
66+
6567
variable (𝕂 : Type*) {m n p : Type*} {n' : m → Type*} {𝔸 : Type*}
6668

6769
namespace Matrix

Mathlib/Analysis/NormedSpace/QuaternionExponential.lean

+2-1
Original file line numberDiff line numberDiff line change
@@ -24,9 +24,10 @@ This file contains results about `exp` on `Quaternion ℝ`.
2424
2525
-/
2626

27-
2827
open scoped Quaternion Nat
2928

29+
open NormedSpace
30+
3031
namespace Quaternion
3132

3233
@[simp, norm_cast]

Mathlib/Analysis/NormedSpace/Spectrum.lean

+2
Original file line numberDiff line numberDiff line change
@@ -47,6 +47,8 @@ This file contains the basic theory for the resolvent and spectrum of a Banach a
4747

4848
open scoped ENNReal NNReal
4949

50+
open NormedSpace -- For `exp`.
51+
5052
/-- The *spectral radius* is the supremum of the `nnnorm` (`‖·‖₊`) of elements in the spectrum,
5153
coerced into an element of `ℝ≥0∞`. Note that it is possible for `spectrum 𝕜 a = ∅`. In this
5254
case, `spectralRadius a = 0`. It is also possible that `spectrum 𝕜 a` be unbounded (though

Mathlib/Analysis/NormedSpace/Star/Exponential.lean

+1
Original file line numberDiff line numberDiff line change
@@ -20,6 +20,7 @@ subtypes `selfAdjoint A` and `unitary A`.
2020
unitaries.
2121
-/
2222

23+
open NormedSpace -- For `exp`.
2324

2425
section Star
2526

Mathlib/Analysis/NormedSpace/Star/Spectrum.lean

+2-2
Original file line numberDiff line numberDiff line change
@@ -21,7 +21,7 @@ section
2121

2222
open scoped Topology ENNReal
2323

24-
open Filter ENNReal spectrum CstarRing
24+
open Filter ENNReal spectrum CstarRing NormedSpace
2525

2626
section UnitarySpectrum
2727

@@ -91,7 +91,7 @@ theorem IsSelfAdjoint.mem_spectrum_eq_re [StarModule ℂ A] {a : A} (ha : IsSelf
9191
(hz : z ∈ spectrum ℂ a) : z = z.re := by
9292
have hu := exp_mem_unitary_of_mem_skewAdjoint ℂ (ha.smul_mem_skewAdjoint conj_I)
9393
let Iu := Units.mk0 I I_ne_zero
94-
have : _root_.exp ℂ (I • z) ∈ spectrum ℂ (_root_.exp ℂ (I • a)) := by
94+
have : NormedSpace.exp ℂ (I • z) ∈ spectrum ℂ (NormedSpace.exp ℂ (I • a)) := by
9595
simpa only [Units.smul_def, Units.val_mk0] using
9696
spectrum.exp_mem_exp (Iu • a) (smul_mem_smul_iff.mpr hz)
9797
exact Complex.ext (ofReal_re _) <| by

Mathlib/Analysis/NormedSpace/TrivSqZeroExt.lean

+2
Original file line numberDiff line numberDiff line change
@@ -38,6 +38,8 @@ variable (𝕜 : Type*) {R M : Type*}
3838

3939
local notation "tsze" => TrivSqZeroExt
4040

41+
open NormedSpace -- For `exp`.
42+
4143
namespace TrivSqZeroExt
4244

4345
section Topology

Mathlib/Analysis/SpecialFunctions/Exponential.lean

+3-3
Original file line numberDiff line numberDiff line change
@@ -53,7 +53,7 @@ We prove most results for an arbitrary field `𝕂`, and then specialize to `
5353
-/
5454

5555

56-
open Filter IsROrC ContinuousMultilinearMap NormedField Asymptotics
56+
open Filter IsROrC ContinuousMultilinearMap NormedField NormedSpace Asymptotics
5757

5858
open scoped Nat Topology BigOperators ENNReal
5959

@@ -216,14 +216,14 @@ theorem hasDerivAt_exp_zero : HasDerivAt (exp 𝕂) (1 : 𝕂) 0 :=
216216

217217
end DerivROrC
218218

219-
theorem Complex.exp_eq_exp_ℂ : Complex.exp = _root_.exp ℂ := by
219+
theorem Complex.exp_eq_exp_ℂ : Complex.exp = NormedSpace.exp ℂ := by
220220
refine' funext fun x => _
221221
rw [Complex.exp, exp_eq_tsum_div]
222222
have : CauSeq.IsComplete ℂ norm := Complex.instIsComplete
223223
exact tendsto_nhds_unique x.exp'.tendsto_limit (expSeries_div_summable ℝ x).hasSum.tendsto_sum_nat
224224
#align complex.exp_eq_exp_ℂ Complex.exp_eq_exp_ℂ
225225

226-
theorem Real.exp_eq_exp_ℝ : Real.exp = _root_.exp ℝ := by
226+
theorem Real.exp_eq_exp_ℝ : Real.exp = NormedSpace.exp ℝ := by
227227
ext x; exact_mod_cast congr_fun Complex.exp_eq_exp_ℂ x
228228
#align real.exp_eq_exp_ℝ Real.exp_eq_exp_ℝ
229229

Mathlib/Analysis/SpecialFunctions/Trigonometric/Series.lean

+1
Original file line numberDiff line numberDiff line change
@@ -20,6 +20,7 @@ In this file we express trigonometric functions in terms of their series expansi
2020
* `Real.hasSum_sin`, `Real.sin_eq_tsum`: `Real.sin` as the sum of an infinite series.
2121
-/
2222

23+
open NormedSpace
2324

2425
open scoped Nat
2526

Mathlib/Combinatorics/Derangements/Exponential.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -17,7 +17,7 @@ The specific lemma is `numDerangements_tendsto_inv_e`.
1717
-/
1818

1919

20-
open Filter
20+
open Filter NormedSpace
2121

2222
open scoped BigOperators
2323

docs/undergrad.yaml

+1-1
Original file line numberDiff line numberDiff line change
@@ -71,7 +71,7 @@ Linear algebra:
7171
examples: ''
7272
Exponential:
7373
endomorphism exponential: ''
74-
matrix exponential: 'exp'
74+
matrix exponential: 'NormedSpace.exp'
7575

7676
# 2.
7777
Group Theory:

0 commit comments

Comments
 (0)