Zulip Chat Archive
Stream: Is there code for X?
Topic: Ring of invariants via typeclass system
Kevin Buzzard (Sep 19 2024 at 23:08):
I have a commutative ring R
, an R
-algebra A
and a (finite) group G
acting on A
. I would like to express the fact that the image of R
in A
is precisely the G
-invariants of A
. This implies SMulCommClass G R A
but it is strictly stronger; SMulCommClass
just means (after a little calculation) that the image of R
in A
is a subset of the G
-invariants.
I don't want to restrict to R : Subring A
because in the applications I'll have things like R=\R
and A=\C
and G being {1,complex conjugation}.
Ideally I would do this entirely within the typeclass framework. Right now I'm carrying around the clunky
variable (hGalois : ∀ (b : B), (∀ (g : G), g • b = b) ↔ ∃ a : A, b = a)
(sorry, B was an A-algebra there)
Daniel Weber (Sep 20 2024 at 02:33):
You can say that docs#MulAction.fixedPoints is equal to the range of algebraMap R A
, but I'm not sure if that's better than what you currently have
Antoine Chambert-Loir (Sep 20 2024 at 06:02):
Define the sub algebra RG of G-invariants and prove that algebraMap A R induces an isomorphism from A to RG?
Filippo A. E. Nuccio (Sep 20 2024 at 07:59):
Have you tried to set up a docs#GaloisInsertion between subgroups of G
and sub-R-algebras of A
and then use Algebra.coe_bot ? Along the lines of docs#LieSubalgebra.gi
Last updated: May 02 2025 at 03:31 UTC