Skip to content

Commit

Permalink
feat(Topology/Algebra): add DiscreteTopology Mˣ (#7028)
Browse files Browse the repository at this point in the history
Add instances for `[DiscreteTopology M] : DiscreteTopology Mᵐᵒᵖ`
and `[DiscreteTopology M] : DiscreteTopology Mˣ`,
as well as additive versions.
  • Loading branch information
urkud committed Sep 8, 2023
1 parent 8908a0a commit 527ecc3
Showing 1 changed file with 13 additions and 1 deletion.
14 changes: 13 additions & 1 deletion Mathlib/Topology/Algebra/Constructions.lean
Expand Up @@ -56,9 +56,13 @@ def opHomeomorph : M ≃ₜ Mᵐᵒᵖ where
#align add_opposite.op_homeomorph AddOpposite.opHomeomorph

@[to_additive]
instance [T2Space M] : T2Space Mᵐᵒᵖ :=
instance instT2Space [T2Space M] : T2Space Mᵐᵒᵖ :=
opHomeomorph.symm.embedding.t2Space

@[to_additive]
instance instDiscreteTopology [DiscreteTopology M] : DiscreteTopology Mᵐᵒᵖ :=
opHomeomorph.symm.embedding.discreteTopology

@[to_additive (attr := simp)]
theorem map_op_nhds (x : M) : map (op : M → Mᵐᵒᵖ) (𝓝 x) = 𝓝 (op x) :=
opHomeomorph.map_nhds_eq x
Expand Down Expand Up @@ -109,6 +113,14 @@ theorem embedding_embedProduct : Embedding (embedProduct M) :=
#align units.embedding_embed_product Units.embedding_embedProduct
#align add_units.embedding_embed_product AddUnits.embedding_embedProduct

@[to_additive]
instance instT2Space [T2Space M] : T2Space Mˣ :=
embedding_embedProduct.t2Space

@[to_additive]
instance instDiscreteTopology [DiscreteTopology M] : DiscreteTopology Mˣ :=
embedding_embedProduct.discreteTopology

@[to_additive] lemma topology_eq_inf :
instTopologicalSpaceUnits =
.induced (val : Mˣ → M) ‹_› ⊓ .induced (fun u ↦ ↑u⁻¹ : Mˣ → M) ‹_› := by
Expand Down

0 comments on commit 527ecc3

Please sign in to comment.