Zulip Chat Archive

Stream: new members

Topic: Glue map from finite intermediate field


Jiang Jiedong (May 20 2024 at 12:32):

Hi everyone,

Is there a theorem in Lean talking about: To define an algebra map on an algebraic field extension (possibly infinite) L/KL/K it suffices to define it on every finite intermediate field F/KF/K compatibly?

The background of this question is a bit lengthy. I am trying to translate the following argument into lean:

Given a field KK, suppose we have defined a subgroup GLG_L of each Gal(L/K)\text{Gal} (L/K) for any finite Galois extension L/KL/K, satisfying that for any tower of finite Galois extensions L/M/KL/M/K, the image of GLG_L in the quotient group Gal(M/K)\text{Gal} (M/K) is exactly GMG_M. (In my case, this GLG_L is exactly the upper numbering ramification group.) In other words, GLG_L is compatible with quotients.

Now I extend the definition of GLG_L to infinite algebraic Galois extensions L/KL/K by setting

GL=limL/F/K,F finite Galois overKGF={sGal(L/K)(sF)GF,L/F/K,F finite Galois overK}.G_L = \varprojlim_{L/F/K, F \text{ finite Galois over} K} G_F \\ = \{ s \in \text{Gal} (L/K) | \, \left(s|_F\right) \in G_F, \forall L/F/K, F \text{ finite Galois over} K\}.

I want to show that this property of "compatible with quotients" still holds for this extended GLG_L, i.e. let L1/L2/KL_1/L_2/K be a tower of (not necessarily finite) Galois extension of fields,

image of GL1 in quotient group Gal(L2/K)=GL2.\text{image of } G_{L_1} \text{ in quotient group Gal} (L_2/K) = G_{L_2} .

Tricky things occur here. Expanding the definition, it suffices to show this key equivalence

sLHS    tGal(L1/K)(i.e. F,tFGF), s.t. tL2=s    F,tFGF, s.t. tFL2F=sL2F    sRHS\begin{align} s \in \text{LHS} & \iff \exist t \in \text{Gal} (L_1/K) (\text{i.e. } \forall F, t|_F \in G_F), \text{ s.t. } t|_{L_2} = s \\ & \iff \forall F, \exists t_F \in G_F, \text{ s.t. } t_F|_{L_2 \cap F} = s|_{L_2 \cap F} \\ & \iff s \in \text{RHS} \end{align}

Here FF is always taken among L1/F/K,F finite Galois over KL_1/F/K, \, F \text{ finite Galois over } K.
The difficulty lies in (2)(2). LHS implies RHS is trivial. For RHS implies LHS, one needs to do the following two things.
(a) To define an element t0t_0 in Gal(L1/K)\text{Gal} (L_1/K) on L, it suffices to find compatible elements tF,0t_{F,0} in each Gal(F/K)\text{Gal} (F/K).
(b) To construct compatible elements tF,0t_{F,0} in each Gal(F/K)\text{Gal} (F/K) from possibly incompatible elements tFt_F, one need to use the fact that finite Galois extensions FF is filtered, and each Gal(F/K)\text{Gal} (F/K) is finite.

Mathematically, the tricky thing here is one must somehow use something "cofiltered limit commutes with finite colimit" like (b) here. I didn't find this category theory theorem CategoryTheory.Limits.FilteredColimitCommutesFiniteLimit in mathlib, although it is claimed in the beginning of Mathlib.CategoryTheory.Filtered.Basic

This is my current attempt. I will be very grateful if anyone has a better roadmap to prove the same goal. Thank you!

Joël Riou (May 20 2024 at 17:57):

The result about the commutation of filtered colimits with finite limits is in the file https://leanprover-community.github.io/mathlib4_docs/Mathlib/CategoryTheory/Limits/FilteredColimitCommutesFiniteLimit.html

Jiang Jiedong said:

Is there a theorem in Lean talking about: To define an algebra map on an algebraic field extension (possibly infinite) L/KL/K it suffices to define it on every finite intermediate field F/KF/K compatibly?

However, I would recommend you try to formulate this result in Lean without using category theory. Then, you should see that it is largely independent from Galois theory.

Andrew Yang (May 20 2024 at 18:48):

I did something similar here


Last updated: May 02 2025 at 03:31 UTC