Zulip Chat Archive
Stream: general
Topic: mul_action
Kenny Lau (Apr 29 2020 at 13:56):
If a group action is a mul_action
, then what is a field action?
Reid Barton (Apr 29 2020 at 13:57):
A vector space?
Johan Commelin (Apr 29 2020 at 13:58):
@Kenny Lau shouldn't you think about group_with_zero
actions first? And what about ring actions?
Reid Barton (Apr 29 2020 at 13:58):
Johan Commelin said:
ring actions?
distrib actions
Kenny Lau (Apr 29 2020 at 14:02):
/- Group action on fields. -/
import group_theory.group_action data.equiv.ring
universes u v
variables (α : Type u) [group α] (β : Type v) [field β]
class group_field_action extends mul_action α β : Type ((max u v)+1) :=
(smul_add : ∀ (g : α) (x y : β), g • (x + y) = g • x + g • y)
(smul_one : ∀ (g : α), (g • 1 : β) = 1)
(smul_mul : ∀ (g : α) (x y : β), g • (x * y) = (g • x) * (g • y))
variables [group_field_action α β]
instance group_field_action.is_ring_hom (g : α) : is_ring_hom (mul_action.to_perm α β g) :=
{ map_one := group_field_action.smul_one g,
map_mul := group_field_action.smul_mul g,
map_add := group_field_action.smul_add g }
def group_field_action.ring_equiv (g : α) : β ≃+* β :=
ring_equiv.of (mul_action.to_perm α β g)
Kenny Lau (Apr 29 2020 at 14:02):
this is my current code
Kenny Lau (Apr 29 2020 at 14:02):
how general can I make this?
Kenny Lau (Apr 29 2020 at 14:02):
monoid on semiring?
Kenny Lau (Apr 29 2020 at 14:02):
based on monoid on add_monoid and monoid on monoid?
Kenny Lau (Apr 29 2020 at 14:02):
what will I call those, mul_add_action and mul_mul_action?
Reid Barton (Apr 29 2020 at 14:02):
Kenny Lau said:
how general can I make this?
A functor between categories
Kenny Lau (Apr 29 2020 at 14:03):
you know what I mean
Kevin Buzzard (Apr 29 2020 at 14:38):
orlando (Apr 29 2020 at 17:10):
Hello perhaps, a generalization is action of on ?
Johan Commelin (Apr 29 2020 at 17:11):
See #2566
Last updated: Dec 20 2023 at 11:08 UTC