Skip to content

Commit

Permalink
unique_stone_cech_extend
Browse files Browse the repository at this point in the history
  • Loading branch information
mapehe committed Apr 15, 2022
1 parent d6a46b7 commit 5c105c8
Showing 1 changed file with 14 additions and 0 deletions.
14 changes: 14 additions & 0 deletions src/topology/stone_cech.lean
Expand Up @@ -262,6 +262,20 @@ ultrafilter_extend_extends f
lemma continuous_stone_cech_extend : continuous (stone_cech_extend hf) :=
continuous_quot_lift _ (continuous_ultrafilter_extend f)

lemma unique_stone_cech_extend {g: stone_cech α → γ} (hg: continuous g)
(hfg: g ∘ stone_cech_unit = (stone_cech_extend hf) ∘ stone_cech_unit):
g = stone_cech_extend hf :=
begin
have h_eq_on: eq_on g (stone_cech_extend hf) (range stone_cech_unit) :=
begin
rw eq_on,
rintros _ ⟨a, ha⟩,
rw [← ha, ← function.comp_apply g stone_cech_unit a],
rw [← function.comp_apply (stone_cech_extend hf) stone_cech_unit a, hfg],
end,
exact continuous.ext_on dense_range_stone_cech_unit hg (continuous_stone_cech_extend hf) h_eq_on,
end

end extension

lemma convergent_eqv_pure {u : ultrafilter α} {x : α} (ux : ↑u ≤ 𝓝 x) : u ≈ pure x :=
Expand Down

0 comments on commit 5c105c8

Please sign in to comment.