Zulip Chat Archive

Stream: Is there code for X?

Topic: cosets / Second isomorphism theorem


Kevin Buzzard (Mar 20 2025 at 08:49):

To develop the theory of Hecke operators for FLT I need what I was taught was the second isomorphism theorem, but to my surprise I've discovered that mathlib's statement of the theorem docs#QuotientGroup.quotientInfEquivProdNormalQuotient was strictly weaker than what I was taught as an undergraduate.

Let GG be a group and let HH and KK be subgroups, with no normality assumption on either (this is why my claim below is different to mathlib's). By H/(HK)H/(H\cap K) I mean the set of left cosets h(HK)h(H\cap K) and by HKHK I mean the set of products {hk:hH,kK}\{hk:h\in H,k\in K\} (note that this is not a group in general, if neither HH nor KK are normal). This set is easily checked to be a union of left cosets hKhK of KK; by HK/KHK/K I mean the set of these left cosets. I was taught that the second isomorphism theorem was the canonical bijection H/(HK)HK/KH/(H\cap K)\cong HK/K sending h(HK)h(H\cap K) to hKhK. And then the rider is that if KK happens to be normal then HKHK is a subgroup and both the things I'm quotienting out by are normal subgroups and the canonical map unsurprisingly preserves multiplication (which is the statement we have in mathlib).

I realised that I didn't even know how to state the version I need. We have HKHK of type Set G as (H : Set G) * (K : Set G) after open scoped Pointwise, but do we even have HK/KHK/K in any form? The \/ symbol only works for groups and in my application HKHK will definitely not be closed under multiplication.


The application is this. Again let HH and KK be subgroups of a (infinite, in my case) group GG (neither of them normal in the application). If GG acts on an additive abelian group AA and if gGg\in G then under the hypothesis that g1HgKg^{-1}Hg\cap K has finite index in g1Hgg^{-1}Hg (and in particular the HH in the previous para is g1Hgg^{-1}Hg here) I claim that there is a map TgT_g from AKA^K (the KK-invariant elements of AA) to AHA^H defined by first decomposing HgKHgK as a finite (by an argument which uses my version of the second isomorphism theorem and the fact that g1HgK/Kg^{-1}HgK/K bijects with HgK/KHgK/K) disjoint union giKg_iK and then sending aa to igi.a\sum_i g_i.a (which is well-defined and in AHA^H if I got all this right; note that it's not yet been formalized). So the #xy of my question is that I want to say "write a subset of GG which is closed under right multiplication by KK as a disjoint union of cosets of KK and choose arbitrary coset representatives" but I would like an idiomatic way to say this if we have such a way (and if not I'll have to make one).

Kevin Buzzard (Mar 20 2025 at 09:34):

Hmm, I guess I could look at subsets of G/KG/K and G/(HK)G/(H\cap K), we have these, hopefully we have the GG-action on them

Edison Xie (Mar 20 2025 at 16:23):

Kevin Buzzard said:

To develop the theory of Hecke operators for FLT I need what I was taught was the second isomorphism theorem, but to my surprise I've discovered that mathlib's statement of the theorem docs#QuotientGroup.quotientInfEquivProdNormalQuotient was strictly weaker than what I was taught as an undergraduate.

Let GG be a group and let HH and KK be subgroups, with no normality assumption on either (this is why my claim below is different to mathlib's). By H/(HK)H/(H\cap K) I mean the set of left cosets h(HK)h(H\cap K) and by HKHK I mean the set of products {hk:hH,kK}\{hk:h\in H,k\in K\} (note that this is not a group in general, if neither HH nor KK are normal). This set is easily checked to be a union of left cosets hKhK of KK; by HK/KHK/K I mean the set of these left cosets. I was taught that the second isomorphism theorem was the canonical bijection H/(HK)HK/KH/(H\cap K)\cong HK/K sending h(HK)h(H\cap K) to hKhK. And then the rider is that if KK happens to be normal then HKHK is a subgroup and both the things I'm quotienting out by are normal subgroups and the canonical map unsurprisingly preserves multiplication (which is the statement we have in mathlib).

I realised that I didn't even know how to state the version I need. We have HKHK of type Set G as (H : Set G) * (K : Set G) after open scoped Pointwise, but do we even have HK/KHK/K in any form? The \/ symbol only works for groups and in my application HKHK will definitely not be closed under multiplication.


The application is this. Again let HH and KK be subgroups of a (infinite, in my case) group GG (neither of them normal in the application). If GG acts on an additive abelian group AA and if gGg\in G then under the hypothesis that g1HgKg^{-1}Hg\cap K has finite index in g1Hgg^{-1}Hg (and in particular the HH in the previous para is g1Hgg^{-1}Hg here) I claim that there is a map TgT_g from AKA^K (the KK-invariant elements of AA) to AHA^H defined by first decomposing HgKHgK as a finite (by an argument which uses my version of the second isomorphism theorem and the fact that g1HgK/Kg^{-1}HgK/K bijects with HgK/KHgK/K) disjoint union giKg_iK and then sending aa to igi.a\sum_i g_i.a (which is well-defined and in AHA^H if I got all this right; note that it's not yet been formalized). So the #xy of my question is that I want to say "write a subset of GG which is closed under right multiplication by KK as a disjoint union of cosets of KK and choose arbitrary coset representatives" but I would like an idiomatic way to say this if we have such a way (and if not I'll have to make one).

would be a great project for the undergrads :joy:


Last updated: May 02 2025 at 03:31 UTC