Zulip Chat Archive

Stream: maths

Topic: Rewriting vs. lifting


Mitchell Lee (Apr 23 2024 at 15:13):

Hi, I was talking to some undergraduate students at the National University of Singapore about how to formalize the theory of Coxeter groups today. We happened upon an idea that I think has the potential to be quite useful, not just for the formalization of Coxeter groups, but for formalization in general. I'm sure this idea is not new, but I have not seen it written down anywhere.

This is best illustrated with an example. Let WW be a Coxeter system with simple generators (si)iB(s_i)_{i \in B} and Coxeter matrix (m(i,i))i,iB(m(i, i'))_{i, i' \in B}. Then we have the following key theorem.

Matsumoto's theorem.

Let si1si=si1sis_{i_1} \cdots s_{i_{\ell}} = s_{i'_1} \cdots s_{i'_\ell} be two reduced expressions for the same element of WW. Then the sequence (i1,,i)(i_1, \ldots, i_\ell) can be transformed into (i1,,i)(i'_1, \ldots, i'_\ell) via a sequence of braid moves. (A braid move on the letters i,iBi, i' \in B, where iii \neq i', changes a contiguous subsequence of length m(i,i)m(i, i') of the form (i,i,i,i,)(i, i', i, i', \ldots) to a sequence of length m(i,i)m(i, i') of the form (i,i,i,i,)(i', i, i', i, \ldots).)

This is a theorem about "rewriting"; that is, changing one string into another by applying a sequence of local moves.

Mitchell Lee (Apr 23 2024 at 15:14):

As useful as this theorem is, it's very difficult to use in a formal setting. For example, suppose that you want to prove that if si1si=si1sis_{i_1} \cdots s_{i_{\ell}} = s_{i'_1} \cdots s_{i'_\ell} are two reduced expressions for the same element of WW, then we have the equality of sets {i1,,i}={i1,,i}\{i_1, \ldots, i_\ell\} = \{i'_1, \ldots, i'_\ell\}. (This is one of the key ingredients in the proof that a parabolic subgroup of a Coxeter group is again a Coxeter group.)

Informally, you would just say "this is a trivial consequence of Matsumoto's theorem". Formally, though, you have to use induction on the number of braid moves used to transform (i1,,i)(i_1, \ldots, i_\ell) to (i1,,i)(i'_1, \ldots, i'_\ell). Then, you need to show that each braid move doesn't change the set of indices, which is really annoying, because you have to split the word into three pieces (the second of which gets affected by the braid move), turn each one into a set, and take the union. Honestly, it seems like a nightmare.

Mitchell Lee (Apr 23 2024 at 15:14):

The solution to this issue is to instead write Matsumoto's theorem in the following equivalent form.

Matsumoto's theorem, equivalent form.

Let MM be a monoid and let f ⁣:BMf \colon B \to M be a function (where BB is the set that indexes the simple reflections of WW). Suppose that for all i,iBi, i' \in B with iii \neq i', we have f(i)f(i)f(i)f(i)=f(i)f(i)f(i)f(i)f(i) f(i') f(i) f(i') \cdots = f(i') f(i) f(i') f(i) \cdots, where there are m(i,i)m(i, i') terms being multiplied on each side of the equation. Then there is a unique function f~ ⁣:WM\tilde f \colon W \to M such that for every reduced word si1sis_{i_1} \cdots s_{i_\ell}, we have f~(si1si)=f(i1)f(i)\tilde f(s_{i_1} \cdots s_{i_\ell}) = f(i_1) \cdots f(i_\ell).

Now, this is a theorem about "lifting"; that is, factoring a function that satisfies a particular property.

Mitchell Lee (Apr 23 2024 at 15:14):

This form is much easier to state and use. (I'm not sure it's easier to prove, but at least you only have to do that once.) To illustrate, let's use it to prove the lemma we had trouble with earlier: if si1si=si1sis_{i_1} \cdots s_{i_{\ell}} = s_{i'_1} \cdots s_{i'_\ell} are two reduced expressions for the same element of WW, then we have the equality of sets {i1,,i}={i1,,i}\{i_1, \ldots, i_\ell\} = \{i'_1, \ldots, i'_\ell\}.

The proof goes as follows. Let MM be the set of all subsets of BB, where the monoid operation is union. For all iBi \in B, let f(i)={i}Mf(i) = \{i\} \in M. Then for all i,iBi, i' \in B with iii \neq i', we have f(i)f(i)f(i)f(i)=f(i)f(i)f(i)f(i)f(i) \cup f(i') \cup f(i) \cup f(i') \cup \cdots = f(i') \cup f(i) \cup f(i') \cup f(i) \cup \cdots, because both sides are equal to {i,i}\{i, i'\}. Hence, the theorem guarantees the existence of a lift f~\tilde f. Finally, we calculate

{i1,,i}=f~(si1si)=f~(si1si)={i1,,i}.\{i_1, \ldots, i_\ell\} = \tilde f(s_{i_1} \cdots s_{i_\ell}) = \tilde f(s_{i'_1} \cdots s_{i'_\ell}) = \{i'_1, \ldots, i'_\ell\}.

This proof method is quite friendly to formalization. Much friendlier than what we were trying to do earlier.

Mitchell Lee (Apr 23 2024 at 15:14):

You can use the same "lifting" form of Matsumoto's theorem to do anything that you could use the "rewriting" form for:

Bruhat order.

Let MM be the set of all subsets of WW, where the monoid operation is pointwise product (i.e. AB={abaA,bB}AB = \{ab \mid a \in A, b \in B\}). Let f(i)={1,si}f(i) = \{1, s_i\}. It is not too difficult to check that this satisfies the hypothesis of Matsumoto's theorem. For all wWw \in W, we have that f~(w)\tilde f(w) is the interval [1,w][1, w] of the (strong) Bruhat order on WW. In fact, this is a reasonable way to define the Bruhat order.

Iwahori-Hecke algebras

Define the Iwahori-Hecke algebra HRH_R by generators, the braid relations, and the quadratic relation. Then, Matsumoto's theorem gives you the elements TwHRT_w \in H_R, and you can show that they form a basis of HRH_R through other means.

Divided difference operators.

Since the divided difference operators i\partial_i satisfy the braid relations of the symmetric group, one can use Matsumoto's theorem to define w\partial_w for all wWw \in W. This is one way to define Schubert polynomials.

Mitchell Lee (Apr 23 2024 at 15:14):

But that's not all. One can show that for any function ff that satisfies the hypotheses of Matsumoto's theorem, the lift f~\tilde f is "almost a monoid homomorphism": that is, f~(1)=1\tilde f(1) = 1 and f~(uv)=f~(u)f~(v)\tilde f(u v) = \tilde f(u) \tilde f(v) for all u,vWu, v \in W such that (uv)=(u)+(v)\ell(uv) = \ell(u) + \ell(v). In fact, this is the defining property of functions obtained through this lifting process. So, by writing Matsumoto's theorem in the lifting form, we now also have a class of functions, the "almost monoid homomorphisms", that we can prove general lemmas about, and we get those lemmas for free in every one of the above examples.

Does anyone have any other examples of theorems that are traditionally stated in a "rewriting" form, but can be instead stated in a "lifting" form? Is there any general design principle to be gleaned here?

Yaël Dillies (Apr 23 2024 at 15:33):

Something like the proof of the ping pong lemma maybe? Not sure I remember correctly

Edward van de Meent (Apr 23 2024 at 15:57):

To me, this problem has a similar "taste" to the work @Floris van Doorn has mentioned in a talk, about notation/api for working with iterated/indexed integrals? the similarities could be very minor though, the talk was a few months ago so i don't remember the details...

Antoine Chambert-Loir (Apr 23 2024 at 17:11):

Mathlib is full of lifting lemmas of this kind. docs#TensorProduct.lift, docs#FreeGroup.lift, docs#SeparationQuotient.lift, etc.

Antoine Chambert-Loir (Apr 23 2024 at 17:13):

IIUC, Matsumoto's theorem goes further: it's not so much about the relations satisfied by the elements of a Coxeter group that about the generators of the canonical morphism from the free group on the simple reflexions to the Coxeter group.

Mitchell Lee (Apr 23 2024 at 22:45):

Yes, there are lifting lemmas in mathlib. But the examples you gave are all explicitly used in the informal literature.

I was asking if there are other theorems that are traditionally stated in the form "A can be rewritten to B using a series of moves" (i.e. in a "syntactic" formulation), but can also be understood as a lifting lemma (i.e. in a "semantic" formulation).


Last updated: May 02 2025 at 03:31 UTC