Skip to content

Commit

Permalink
chore(Topology): Fintype -> Finite (#10262)
Browse files Browse the repository at this point in the history
  • Loading branch information
urkud committed Feb 5, 2024
1 parent a12f60d commit fbee97e
Show file tree
Hide file tree
Showing 3 changed files with 5 additions and 5 deletions.
6 changes: 3 additions & 3 deletions Mathlib/Topology/Algebra/Module/FiniteDimension.lean
Expand Up @@ -270,7 +270,7 @@ instance LinearMap.continuousLinearMapClassOfFiniteDimensional [T2Space E] [Fini
This is the key fact which makes all linear maps from a T2 finite dimensional TVS over such a field
continuous (see `LinearMap.continuous_of_finiteDimensional`), which in turn implies that all
norms are equivalent in finite dimensions. -/
theorem continuous_equivFun_basis [T2Space E] {ι : Type*} [Fintype ι] (ξ : Basis ι 𝕜 E) :
theorem continuous_equivFun_basis [T2Space E] {ι : Type*} [Finite ι] (ξ : Basis ι 𝕜 E) :
Continuous ξ.equivFun :=
haveI : FiniteDimensional 𝕜 E := of_fintype_basis ξ
ξ.equivFun.toLinearMap.continuous_of_finiteDimensional
Expand Down Expand Up @@ -433,7 +433,7 @@ namespace Basis

set_option linter.uppercaseLean3 false

variable {ι : Type*} [Fintype ι] [T2Space E]
variable {ι : Type*} [Finite ι] [T2Space E]

/-- Construct a continuous linear map given the value at a finite basis. -/
def constrL (v : Basis ι 𝕜 E) (f : ι → F) : E →L[𝕜] F :=
Expand Down Expand Up @@ -465,7 +465,7 @@ lemma equivFunL_symm_apply_repr (v : Basis ι 𝕜 E) (x : E) :
v.equivFunL.symm_apply_apply x

@[simp]
theorem constrL_apply (v : Basis ι 𝕜 E) (f : ι → F) (e : E) :
theorem constrL_apply {ι : Type*} [Fintype ι] (v : Basis ι 𝕜 E) (f : ι → F) (e : E) :
v.constrL f e = ∑ i, v.equivFun e i • f i :=
v.constr_apply_fintype 𝕜 _ _
#align basis.constrL_apply Basis.constrL_apply
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Topology/Bases.lean
Expand Up @@ -470,7 +470,7 @@ theorem isSeparable_iUnion {ι : Type*} [Countable ι] {s : ι → Set α}
exact (h'c i).trans (closure_mono (subset_iUnion _ i))
#align topological_space.is_separable_Union TopologicalSpace.isSeparable_iUnion

lemma isSeparable_pi {ι : Type*} [Fintype ι] {α : ∀ (_ : ι), Type*} {s : ∀ i, Set (α i)}
lemma isSeparable_pi {ι : Type*} [Finite ι] {α : ι → Type*} {s : ∀ i, Set (α i)}
[∀ i, TopologicalSpace (α i)] (h : ∀ i, IsSeparable (s i)) :
IsSeparable {f : ∀ i, α i | ∀ i, f i ∈ s i} := by
choose c c_count hc using h
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Topology/Bornology/Constructions.lean
Expand Up @@ -20,7 +20,7 @@ open Set Filter Bornology Function

open Filter

variable {α β ι : Type*} {π : ι → Type*} [Fintype ι] [Bornology α] [Bornology β]
variable {α β ι : Type*} {π : ι → Type*} [Finite ι] [Bornology α] [Bornology β]
[∀ i, Bornology (π i)]

instance Prod.instBornology : Bornology (α × β) where
Expand Down

0 comments on commit fbee97e

Please sign in to comment.