Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 627bd0c

Browse files
committed
chore(topology/basic): use finite in locally_finite_of_finite (#15181)
Rename `locally_finite_of_fintype` to `locally_finite_of_finite`, use `[finite]` instead of `[fintype]`.
1 parent 7f837db commit 627bd0c

File tree

2 files changed

+2
-2
lines changed

2 files changed

+2
-2
lines changed

src/topology/basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1191,7 +1191,7 @@ lemma locally_finite.point_finite {f : β → set α} (hf : locally_finite f) (x
11911191
{b | x ∈ f b}.finite :=
11921192
let ⟨t, hxt, ht⟩ := hf x in ht.subset $ λ b hb, ⟨x, hb, mem_of_mem_nhds hxt⟩
11931193

1194-
lemma locally_finite_of_fintype [fintype β] (f : β → set α) : locally_finite f :=
1194+
lemma locally_finite_of_finite [finite β] (f : β → set α) : locally_finite f :=
11951195
assume x, ⟨univ, univ_mem, to_finite _⟩
11961196

11971197
lemma locally_finite.subset

src/topology/paracompact.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -112,7 +112,7 @@ begin
112112
rcases compact_univ.elim_finite_subcover _ ho hu.ge with ⟨T, hT⟩,
113113
have := hT, simp only [subset_def, mem_Union] at this,
114114
choose i hiT hi using λ x, this x (mem_univ x),
115-
refine ⟨(T : set ι), λ t, s t, λ t, ho _, _, locally_finite_of_fintype _, λ t, ⟨t, subset.rfl⟩⟩,
115+
refine ⟨(T : set ι), λ t, s t, λ t, ho _, _, locally_finite_of_finite _, λ t, ⟨t, subset.rfl⟩⟩,
116116
simpa only [Union_coe_set, ← univ_subset_iff]
117117
end
118118

0 commit comments

Comments
 (0)