Skip to content

Commit 1dc9adf

Browse files
committed
chore(NormedSpace/Exponential): Fintype → Finite (#10260)
1 parent 28c0092 commit 1dc9adf

File tree

1 file changed

+4
-4
lines changed

1 file changed

+4
-4
lines changed

Mathlib/Analysis/NormedSpace/Exponential.lean

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -569,20 +569,20 @@ theorem _root_.Prod.snd_exp [CompleteSpace 𝔹] (x : 𝔸 × 𝔹) : (exp 𝕂
569569
#align prod.snd_exp Prod.snd_exp
570570

571571
@[simp]
572-
theorem _root_.Pi.exp_apply {ι : Type*} {𝔸 : ι → Type*} [Fintype ι] [∀ i, NormedRing (𝔸 i)]
572+
theorem _root_.Pi.exp_apply {ι : Type*} {𝔸 : ι → Type*} [Finite ι] [∀ i, NormedRing (𝔸 i)]
573573
[∀ i, NormedAlgebra 𝕂 (𝔸 i)] [∀ i, CompleteSpace (𝔸 i)] (x : ∀ i, 𝔸 i) (i : ι) :
574574
exp 𝕂 x i = exp 𝕂 (x i) :=
575+
let ⟨_⟩ := nonempty_fintype ι
575576
map_exp _ (Pi.evalRingHom 𝔸 i) (continuous_apply _) x
576-
-- porting note: Lean can now handle Π-types in type class inference!
577577
#align pi.exp_apply Pi.exp_apply
578578

579-
theorem _root_.Pi.exp_def {ι : Type*} {𝔸 : ι → Type*} [Fintype ι] [∀ i, NormedRing (𝔸 i)]
579+
theorem _root_.Pi.exp_def {ι : Type*} {𝔸 : ι → Type*} [Finite ι] [∀ i, NormedRing (𝔸 i)]
580580
[∀ i, NormedAlgebra 𝕂 (𝔸 i)] [∀ i, CompleteSpace (𝔸 i)] (x : ∀ i, 𝔸 i) :
581581
exp 𝕂 x = fun i => exp 𝕂 (x i) :=
582582
funext <| Pi.exp_apply 𝕂 x
583583
#align pi.exp_def Pi.exp_def
584584

585-
theorem _root_.Function.update_exp {ι : Type*} {𝔸 : ι → Type*} [Fintype ι] [DecidableEq ι]
585+
theorem _root_.Function.update_exp {ι : Type*} {𝔸 : ι → Type*} [Finite ι] [DecidableEq ι]
586586
[∀ i, NormedRing (𝔸 i)] [∀ i, NormedAlgebra 𝕂 (𝔸 i)] [∀ i, CompleteSpace (𝔸 i)] (x : ∀ i, 𝔸 i)
587587
(j : ι) (xj : 𝔸 j) :
588588
Function.update (exp 𝕂 x) j (exp 𝕂 xj) = exp 𝕂 (Function.update x j xj) := by

0 commit comments

Comments
 (0)