Skip to content

Commit

Permalink
feat(topology/algebra/uniform_group): uniform_group is preserved by…
Browse files Browse the repository at this point in the history
… Inf and comap (#14889)

This is the uniform version of #11720
  • Loading branch information
ADedecker committed Jul 8, 2022
1 parent 6eeb941 commit ba9f346
Show file tree
Hide file tree
Showing 2 changed files with 36 additions and 1 deletion.
35 changes: 35 additions & 0 deletions src/topology/algebra/uniform_group.lean
Expand Up @@ -145,6 +145,41 @@ namespace subgroup

end subgroup

section lattice_ops

variables [group β]

@[to_additive] lemma uniform_group_Inf {us : set (uniform_space β)}
(h : ∀ u ∈ us, @uniform_group β u _) :
@uniform_group β (Inf us) _ :=
{ uniform_continuous_div := uniform_continuous_Inf_rng (λ u hu, uniform_continuous_Inf_dom₂ hu hu
(@uniform_group.uniform_continuous_div β u _ (h u hu))) }

@[to_additive] lemma uniform_group_infi {ι : Sort*} {us' : ι → uniform_space β}
(h' : ∀ i, @uniform_group β (us' i) _) :
@uniform_group β (⨅ i, us' i) _ :=
by {rw ← Inf_range, exact uniform_group_Inf (set.forall_range_iff.mpr h')}

@[to_additive] lemma uniform_group_inf {u₁ u₂ : uniform_space β}
(h₁ : @uniform_group β u₁ _) (h₂ : @uniform_group β u₂ _) :
@uniform_group β (u₁ ⊓ u₂) _ :=
by {rw inf_eq_infi, refine uniform_group_infi (λ b, _), cases b; assumption}

@[to_additive] lemma uniform_group_comap {γ : Type*} [group γ] {u : uniform_space γ}
[uniform_group γ] {F : Type*} [monoid_hom_class F β γ] (f : F) :
@uniform_group β (u.comap f) _ :=
{ uniform_continuous_div :=
begin
letI : uniform_space β := u.comap f,
refine uniform_continuous_comap' _,
simp_rw [function.comp, map_div],
change uniform_continuous ((λ p : γ × γ, p.1 / p.2) ∘ (prod.map f f)),
exact uniform_continuous_div.comp
(uniform_continuous_comap.prod_map uniform_continuous_comap),
end }

end lattice_ops

section
variables (α)

Expand Down
2 changes: 1 addition & 1 deletion src/topology/uniform_space/basic.lean
Expand Up @@ -1158,7 +1158,7 @@ begin
exact comap_mono hu
end

lemma uniform_continuous_iff {α β} [uα : uniform_space α] [uβ : uniform_space β] {f : α → β} :
lemma uniform_continuous_iff {α β} {uα : uniform_space α} {uβ : uniform_space β} {f : α → β} :
uniform_continuous f ↔ uα ≤ uβ.comap f :=
filter.map_le_iff_le_comap

Expand Down

0 comments on commit ba9f346

Please sign in to comment.