Skip to content

Commit

Permalink
feat: port Topology.Algebra.Module.Basic (#2983)
Browse files Browse the repository at this point in the history
Co-authored-by: Moritz Doll <moritz.doll@googlemail.com>
Co-authored-by: Yury G. Kudryashov <urkud@urkud.name>
Co-authored-by: Komyyy <pol_tta@outlook.jp>
Co-authored-by: Yury Kudryashov <urkud@urkud.name>
Co-authored-by: ChrisHughes24 <chrishughes24@gmail.com>
Co-authored-by: Parcly Taxel <reddeloostw@gmail.com>
  • Loading branch information
6 people committed Apr 4, 2023
1 parent 56c1ca9 commit 2dd4be1
Show file tree
Hide file tree
Showing 3 changed files with 2,824 additions and 1 deletion.
1 change: 1 addition & 0 deletions Mathlib.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1594,6 +1594,7 @@ import Mathlib.Topology.Algebra.InfiniteSum.Order
import Mathlib.Topology.Algebra.InfiniteSum.Real
import Mathlib.Topology.Algebra.InfiniteSum.Ring
import Mathlib.Topology.Algebra.Localization
import Mathlib.Topology.Algebra.Module.Basic
import Mathlib.Topology.Algebra.Monoid
import Mathlib.Topology.Algebra.MulAction
import Mathlib.Topology.Algebra.Nonarchimedean.Basic
Expand Down
10 changes: 9 additions & 1 deletion Mathlib/Topology/Algebra/ConstMulAction.lean
Original file line number Diff line number Diff line change
Expand Up @@ -171,7 +171,7 @@ instance Units.continuousConstSMul : ContinuousConstSMul Mˣ α

@[to_additive]
theorem smul_closure_subset (c : M) (s : Set α) : c • closure s ⊆ closure (c • s) :=
((Set.mapsTo_image _ _).closure <| continuous_id.const_smul c).image_subset
((Set.mapsTo_image _ _).closure <| continuous_const_smul c).image_subset
#align smul_closure_subset smul_closure_subset
#align vadd_closure_subset vadd_closure_subset

Expand All @@ -182,6 +182,14 @@ theorem smul_closure_orbit_subset (c : M) (x : α) :
#align smul_closure_orbit_subset smul_closure_orbit_subset
#align vadd_closure_orbit_subset vadd_closure_orbit_subset

theorem isClosed_setOf_map_smul [Monoid N] (α β) [MulAction M α] [MulAction N β]
[TopologicalSpace β] [T2Space β] [ContinuousConstSMul N β] (σ : M → N) :
IsClosed { f : α → β | ∀ c x, f (c • x) = σ c • f x } := by
simp only [Set.setOf_forall]
exact isClosed_interᵢ fun c => isClosed_interᵢ fun x =>
isClosed_eq (continuous_apply _) ((continuous_apply _).const_smul _)
#align is_closed_set_of_map_smul isClosed_setOf_map_smulₓ

end Monoid

section Group
Expand Down
Loading

0 comments on commit 2dd4be1

Please sign in to comment.