Zulip Chat Archive
Stream: Is there code for X?
Topic: Continuous actions
Christian Merten (Dec 10 2023 at 22:37):
As already discussed here: https://leanprover.zulipchat.com/#narrow/stream/217875-Is-there-code-for-X.3F/topic/Finite.20colimits.20in.20Action, I would like to have the category of continuous actions. I now propose the possibly naive approach:
import Mathlib.RepresentationTheory.Action.Basic
import Mathlib.Topology.Constructions
import Mathlib.Topology.Algebra.MulAction
universe u v
open CategoryTheory
variable (V : Type (u+1)) [LargeCategory V] (G : MonCat.{u}) [ConcreteCategory V]
instance (X : Action V G) : MulAction G ((forget V).obj X.V) where
smul g x := (forget V).map (X.ρ g) x
one_smul x := by
show (forget V).map (X.ρ 1) x = x
simp only [Action.ρ_one, FunctorToTypes.map_id_apply]
mul_smul g h x := by
show (forget V).map (X.ρ (g * h)) x = ((forget V).map (X.ρ h) ≫ (forget V).map (X.ρ g)) x
rw [←Functor.map_comp, map_mul]
rfl
variable [∀ (X : Action V G), TopologicalSpace ((forget V).obj X.V)]
[TopologicalSpace (G : Type u)]
def cont (X : Action V G) : Prop := ContinuousSMul G ((forget V).obj X.V)
def ContAction : Type (u+1) := FullSubcategory (cont V G)
instance : Category (ContAction V G) := FullSubcategory.category (cont V G)
This only works for concrete categories, which seems to be necessary to even write down the map .
Is it a bad idea to have this MulAction
instance? This might cause issues when docs#Action.ofMulAction is used to obtain an element X : Action (Type u) G
. One could also drop the instance and just copy the definition of ContinuousSMul
specialized to this situation.
Do you have any thoughts on this?
Last updated: Dec 20 2023 at 11:08 UTC