Datasets:
Tasks:
Text Generation
Modalities:
Text
Sub-tasks:
language-modeling
Languages:
English
Size:
100K - 1M
License:
/- | |
Copyright (c) 2021 Nicolò Cavalleri. All rights reserved. | |
Released under Apache 2.0 license as described in the file LICENSE. | |
Authors: Nicolò Cavalleri | |
-/ | |
import topology.homeomorph | |
/-! | |
# Topological space structure on the opposite monoid and on the units group | |
In this file we define `topological_space` structure on `Mᵐᵒᵖ`, `Mᵃᵒᵖ`, `Mˣ`, and `add_units M`. | |
This file does not import definitions of a topological monoid and/or a continuous multiplicative | |
action, so we postpone the proofs of `has_continuous_mul Mᵐᵒᵖ` etc till we have these definitions. | |
## Tags | |
topological space, opposite monoid, units | |
-/ | |
variables {M X : Type*} | |
open filter | |
open_locale topological_space | |
namespace mul_opposite | |
/-- Put the same topological space structure on the opposite monoid as on the original space. -/ | |
topological_space.induced (unop : Mᵐᵒᵖ → M) ‹_› | |
variables [topological_space M] | |
continuous_induced_dom | |
continuous_induced_rng.2 continuous_id | |
⟨λ x y h, separated_by_continuous mul_opposite.continuous_unop $ unop_injective.ne h⟩ | |
/-- `mul_opposite.op` as a homeomorphism. -/ | |
def op_homeomorph : M ≃ₜ Mᵐᵒᵖ := | |
{ to_equiv := op_equiv, | |
continuous_to_fun := continuous_op, | |
continuous_inv_fun := continuous_unop } | |
op_homeomorph.map_nhds_eq x | |
op_homeomorph.symm.map_nhds_eq x | |
op_homeomorph.comap_nhds_eq x | |
op_homeomorph.symm.comap_nhds_eq x | |
end mul_opposite | |
namespace units | |
open mul_opposite | |
variables [topological_space M] [monoid M] | |
/-- The units of a monoid are equipped with a topology, via the embedding into `M × M`. -/ | |
topological_space.induced (embed_product M) prod.topological_space | |
⟨inducing_embed_product, embed_product_injective M⟩ | |
continuous_induced_dom | |
(@continuous_embed_product M _ _).fst | |
end units | |