Zulip Chat Archive

Stream: Is there code for X?

Topic: continuous semi-algebra maps


Kevin Buzzard (Jan 07 2025 at 14:14):

If KK and LL are number fields with LL a KK-algebra, and if ww is a place of LL dividing a place vv of KK (i.e. vv is the pullback of ww to KK), then there is a canonical inclusion of the completions KvLwK_v\to L_w extending the canonical map KLK\to L. This map is a continuous semilinear algebra morphism and my instinct is that what I've just said is by far the nicest way to express what is going on. But we don't even have semilinear algebra morphisms in Lean, let alone continuous ones.

Should I encourage someone to set up all the machinery of semilinear algebra maps, semilinear algebra map classes, continuous semilinear algebra maps and continuous semilinear algebra map classes? (or am I blind and we have some or all of these already?) Could we envisage having all of this in mathlib? It's probably worth flagging that semilinear algebra maps are what looks to me like a nice way of encoding commutative squares where the vertical maps are algebraMap (which is often the case, for example in the AKLB set-up we have K an A-algebra and L a B-algebra, and we're currently expressing commutativity of the square with two IsScalarTower instances).

Eric Wieser (Jan 07 2025 at 14:34):

Semilinear algebra maps don't work so well for when there are two connected commutative squares, right?

Michael Stoll (Jan 07 2025 at 15:04):

What is the "semi" here in "semilinear"?

Kevin Buzzard (Jan 07 2025 at 15:25):

Eric Wieser said:

Semilinear algebra maps don't work so well for when there are two connected commutative squares, right?

We have docs#LinearMap.comp which is composition of semilinear maps, I can't imagine that demanding that the top maps preserve multiplication will be any different? Or are you stacking the squares vertically? In the examples coming from adeles the stacking is horizontal like in the linear map case.

Kevin Buzzard (Jan 07 2025 at 15:25):

Michael Stoll said:

What is the "semi" here in "semilinear"?

Sorry, I realise I didn't even mention that we already have semilinear maps and continuous semilinear maps in mathlib. I guess I mean "semialgebra maps"?

The map KvLwK_v\to L_w is semilinear in the sense that the square with this on the top and KLK\to L on the bottom commutes. See the definition of docs#LinearMap (note the presence of two base rings and notation →ₛₗ[σ]). See https://arxiv.org/abs/2202.05360 for the story of the formalization.

Kevin Buzzard (Jan 07 2025 at 15:28):

In FLT at the minute, in the nonarch case, I'm expressing that the square with KvLwK_v\to L_w and KLK\to L commutes by artificially making LwL_w into a KK-algebra (it's already an LL-algebra), demanding the IsScalarTower instance making the triangle commute, and then saying that the map is KK-linear. For this to even make sense we have to have LL a KK-algebra rather than just a morphism of rings. It just occurred to me today when thinking about the infinite case that a much more conceptual way of stating this would be just by showing that the map KvLwK_v\to L_w is semilinear wrt KLK\to L.

Jireh Loreaux (Jan 07 2025 at 17:42):

I was hoping we could get away without semilinear algebra maps, but since you have a use case, then I think we should develop them. There is also another use case I know about (the modular conjugation operator in Tomita-Takesaki theory), but it's sufficiently specialized that it probably could be it's own thing if semilinear algebra maps weren't need elsewhere.

Antoine Chambert-Loir (Jan 08 2025 at 17:18):

When I had developed the semilinear maps of actions, I had refactored the semilinear maps of modules, but I had noticed that the semi-linear extension stopped just before the algebra map. Of course, the docs#IsScalarTower is more or less playing the same game and the interaction between the two will have to be clarified.

Kevin Buzzard (Jan 08 2025 at 17:29):

One difference is that if I want different maps KLK\to L then I'm in trouble with IsScalarTower because it wants [Algebra K L] (well, it wants SMul K L but in practice this is coming from Alegbra K L).


Last updated: May 02 2025 at 03:31 UTC