File tree Expand file tree Collapse file tree 1 file changed +0
-8
lines changed Expand file tree Collapse file tree 1 file changed +0
-8
lines changed Original file line number Diff line number Diff line change @@ -39,14 +39,6 @@ theorem point_finite (hf : LocallyFinite f) (x : X) : { b | x ∈ f b }.Finite :
3939 ht.subset fun _b hb => ⟨x, hb, mem_of_mem_nhds hxt⟩
4040#align locally_finite.point_finite LocallyFinite.point_finite
4141
42- @[to_additive]
43- theorem exists_finset_mulSupport_eq {M : Type *} [CommMonoid M] {ρ : ι → X → M}
44- (hρ : LocallyFinite fun i ↦ mulSupport <| ρ i) (x₀ : X) :
45- ∃ I : Finset ι, (mulSupport fun i ↦ ρ i x₀) = I := by
46- use (hρ.point_finite x₀).toFinset
47- rw [Finite.coe_toFinset]
48- exact rfl
49-
5042protected theorem subset (hf : LocallyFinite f) (hg : ∀ i, g i ⊆ f i) : LocallyFinite g := fun a =>
5143 let ⟨t, ht₁, ht₂⟩ := hf a
5244 ⟨t, ht₁, ht₂.subset fun i hi => hi.mono <| inter_subset_inter (hg i) Subset.rfl⟩
You can’t perform that action at this time.
0 commit comments