Zulip Chat Archive
Stream: Equational
Topic: Equation 65 -> left cancellability
Daniel Weber (Oct 07 2024 at 04:20):
I attempted to think of Equation 65 -> Equation 359 (x = y ◇ (x ◇ (y ◇ x)) -> x ◇ x = (x ◇ x) ◇ x) for a couple of hours, but couldn't think of anything successful.
My first attempt was to look at sextuples of natural numbers, and define the operation as "rotate the RHS by 2, and if the XORs of the numbers in the LHS and in the RHS are different then XOR to the all numbers on the RHS the xor of all numbers on the LHS". The idea here that the XOR is an invariant - the XOR of the output is the XOR of the LHS, and using it the involution of "XOR some values depending on y
to all values" can only fire for y
, not for x
. The problem with this, of course, is that the interesting part doesn't activate for (x ◇ x) ◇ x
, so it satisfies equation 359.
Then I wanted to generalize it, by using the fact that the LHS isn't rotated---define some compatibility relation, such that compatible(y, x ◇ (y ◇ x)) ↔ compatible(y, x)
and compatible(x, y ◇ x)
, and then define the operation differently based on whether the LHS and the RHS are compatible. The problem with this is that for it to be interesting we need ¬ compatible(x ◇ x, x)
, and I'm not sure how to get that.
One thing I thought of is finding a triple of functions such that , but not the other way round . I have a vague intuition that this could be helpful, as pairs of functions such that had been useful for other infinite models, but I'm not sure.
Terence Tao (Oct 07 2024 at 04:53):
It seems to me that the linear operation x ◇ y = ω y
, where ω
is a cube root of unity in the ambient field, should establish the anti-implication, no? But then it should have been picked up by the large linear magma sweep we just did, which is odd.
(Just to record my thought process on how I found this example. I postulated that there was some unary operation L
on the magma so that x ◇ (y ◇ x) = L(x)
and x = y ◇ L(x)
, in order to break up the hypothesis 65 into simpler pieces. The second law forces L
to be injective. Replacing x
with L(x)
in the first law got me to L(x) ◇ x = L^2(x)
, and replacing x
with L(x)
again then got me to x = L^3(x)
. At this point I realized I should try L
being multiplication by a cube root of unity, leading to the above example.)
EDIT: oh, wait, this example also obeys 359, so it isn't a counterexample. Ah, not as easy as it looks...
Terence Tao (Oct 07 2024 at 05:05):
OK, trying again, this time with a general linear operation x ◇ y = ax+by
. If I have calculated things correctly, Equation 65 becomes the system a(1+b^2)=0, b(a+b^2)=1
, and Equation 359 becomes a(a+b-1)=0
. Oh, interesting, here it does seem that again the former implies the latter. If a=0
this is clear, otherwise we have 1+b^2=0
and b(a+b^2)=1
, and on multiplying the latter by b
and substituting b^2=-1
we get after some algebra a+b-1=0
. OK, this explains why this wasn't picked up by the linear magma sweep.
Zoltan A. Kocsis (Z.A.K.) (Oct 07 2024 at 06:15):
This is the "sibling" of the 65->3862 potential implication that I proposed in this thread, right? I don't have access to my notes right now but IIRC 65 and 359 together imply 3862, so it'd resolve that too.
Daniel Weber (Oct 07 2024 at 07:32):
Could you explain the proof that the implication holds on finite magmas? I imagine that might guide searching for counterexamples
Daniel Weber (Oct 07 2024 at 10:20):
Here's another idea I had:
We define an inductive type with three constructors, t : type -> type -> type
, pair : type -> type -> type
and nil : type
. We write (a, b)
for pair a b
, t_x(a)
for t x a
and t_x(a, b)
for t_x(pair a b)
.
We now start with basic definition a * b = (a, b)
, and each time add exceptions, the latest applicable definition is the one that applies, and the idea is to eventually get a model where 65 holds. First we add b * (a, b) = t_a(b)
and a * t_a(b) = b
.
Now b * ((a, b) * (b * (a, b))) = b * ((a, b) * t_a(b)) != (a, b)
, so we add (a, b) * t_a(b) = t_b(a, b)
.
Now a * (t_a(b) * (a * t_a(b))) = a * (t_a(b) * b) != t_a(b)
, so we add t_a(b) * b = t_a(t_a(b))
.
Then (a,b) * (t_a(b) * t_b(a, b)) != t_a(b)
, so we add t_a(b) * t_b(a,b) = t_{a,b}(t_a(b))
.
This can continue manually, but is probably better done using a computer (either semi or fully automatically), until we either finish, or maybe spot a pattern and generalize it.
Does this seem likely to work? Is there a better inductive type/basic definitions? Perhaps more constructors will be better?
Daniel Weber (Oct 07 2024 at 12:18):
I think that's actually just equality saturation, which probably doesn't finish in a sensible number of steps, as vampire would've found that, but perhaps we could see some pattern to the equations
Daniel Weber (Oct 07 2024 at 15:30):
Apparently (a, b) * t_a(b) = t_b(a, b)
is too strong of an assumption, it implies 359
Terence Tao (Oct 07 2024 at 15:37):
OK, here is yet another attempt at creating a counterexample, inspired by @Daniel Weber 's triple function idea.
Let be a triple of functions to be chosen later. We extend this periodically mod 3, thus . Now consider the magma with operation
Then we have
and
so 359 is certainly false. On the other hand,
so if we can solve the equations
then we get a counterexample.
Oh, but we can just take all the to be the identity! And to be trivial! So, um, it seems that a really simple counterexample is with operation . That was embarrassingly obvious. But perhaps the more general construction above will be helpful for other problems.
The broader metatheorem seems to be: if the hypothesis is with both ending in the same letter, and whose lengths are equal modulo , then all equations implied by this hypothesis have to have the same property. Proof: use the operation on . I'll add that metatheorem to the blueprint later today.
But it does raise an obvious TODO: study affine magmas and see if they can clear out a chunk of the remaining implications.
Daniel Weber (Oct 07 2024 at 15:39):
doesn't work, it satisfies
Daniel Weber (Oct 07 2024 at 15:42):
The problem is that , but I think the functional equation could still potentially be solved to generate a counterexample
Terence Tao (Oct 07 2024 at 15:42):
Argh! Can't believe I made the same mistake three times in a row. I should have computed
so actually one needs to solve the system
which looks doable (but I haven't checked details, maybe I made another mistake).
Daniel Weber (Oct 07 2024 at 15:44):
Sadly this is impossible,
Daniel Weber (Oct 07 2024 at 15:52):
A potential approach using Vampire is to try and add some equations (and maybe some pairs of equations) in hopes that they might not imply Equation 359 but still limit the search space enough for Vampire to find a saturation
Daniel Weber (Oct 07 2024 at 15:59):
Is it theoretically possible that there's a false implication which we can't disprove in ZFC?
Pace Nielsen (Oct 07 2024 at 16:08):
Using a map of the form x⋄y=ax+by+c, leads to the set of equations ba+b^3=1, a+b^2a=0, and a^2+ab\neq a. It turns out these are inconsistent over noncommutative rings. So no affine map with work over coefficients from a ring.
Pace Nielsen (Oct 07 2024 at 16:13):
Daniel Weber said:
Is it theoretically possible that there's a false implication which we can't disprove in ZFC?
Yes, it was shown in the literature that whether or not an equation implies x=y is algorithmically undecidable.
Terence Tao (Oct 07 2024 at 16:15):
Daniel Weber said:
Is it theoretically possible that there's a false implication which we can't disprove in ZFC?
That's a good question. I believe there finite systems of equations, for which it is undecidable in ZFC whether they imply some other equation, but I don't know the literature well. Actually it will be good to sort this out, this needs to be mentioned in the paper.
Shame that the functional and the ring-theoretic approaches now seem fairly conclusively ruled out. On the other hand, perhaps this should be viewed as evidence that the implication is in fact true? We've now constructed a reasonably diverse set of models to 65 and they all "accidentally" happen to satisfy 359 as well. This is beginning to look like it's not a coincidence... perhaps the above arguments can somehow be deconstructed for clues on how to get from 65 to 359, e.g., by identifying some intermediate assertion that also seems to be true for all the models?
EDIT: we should also test the above models on the other unresolved potential consequences 614, 817, 1426, 1491, 3862, 4065 of 65. And maybe try to work out the logical relations between these statements assuming 65 as an ambient hypothesis. We might be trying to work on the hardest implication, despite it being the shortest unresolved one.
Terence Tao (Oct 07 2024 at 16:21):
@Vlad Tsyrklevich Is it easy to get Graphiti to do a Hasse diagram of all the statements that are either implied by, or potentially implied by, a given statement such as 65?
EDIT: Oh, it is!
Terence Tao (Oct 07 2024 at 16:25):
From the diagram it seems we should test both the ring-theoretic and the function-theoretic constructions against 1491 first.
Terence Tao (Oct 07 2024 at 16:26):
(But it would be nice to have the ability to generate this graph in one click from the Equation Explorer page for 65. I did it manually by entering in all the potential consequences of 65.)
Daniel Weber (Oct 07 2024 at 16:27):
Terence Tao said:
Daniel Weber said:
Is it theoretically possible that there's a false implication which we can't disprove in ZFC?
That's a good question. I believe there finite systems of equations, for which it is undecidable in ZFC whether they imply some other equation, but I don't know the literature well. Actually it will be good to sort this out, this needs to be mentioned in the paper.
Shame that the functional and the ring-theoretic approaches now seem fairly conclusively ruled out. On the other hand, perhaps this should be viewed as evidence that the implication is in fact true? We've now constructed a reasonably diverse set of models to 65 and they all "accidentally" happen to satisfy 359 as well. This is beginning to look like it's not a coincidence... perhaps the above arguments can somehow be deconstructed for clues on how to get from 65 to 359, e.g., by identifying some intermediate assertion that also seems to be true for all the models?
EDIT: we should also test the above models on the other unresolved potential consequences 614, 817, 1426, 1491, 3862, 4065 of 65. And maybe try to work out the logical relations between these statements assuming 65 as an ambient hypothesis. We might be trying to work on the hardest implication, despite it being the shortest unresolved one.
I still think that this is false, but all the models we managed to think of are too nice for it to fail. In particular, the magma being left cancellative implies 359, as does f_y(x) = x * (y * x)
being surjective for all y
Terence Tao (Oct 07 2024 at 16:47):
Do you have proofs of these assertions written up somewhere? They might provide further clues.
The function model at least doesn't have surjectivity of f_y, and could potentially be not left-cancellative if the functions involved are not injective. So I hold out some hope that some more sophisticated version of the model (e.g., where depends in some relatively mild way on ) might still work.
EDIT: the new system seems to be
Daniel Weber (Oct 07 2024 at 17:20):
Terence Tao said:
Do you have proofs of these assertions written up somewhere? They might provide further clues.
[...]
Vampire proved them and I'm not at home right now, I'll send them in a couple of hours
Vlad Tsyrklevich (Oct 07 2024 at 17:28):
Terence Tao said:
(But it would be nice to have the ability to generate this graph in one click from the Equation Explorer page for 65. I did it manually by entering in all the potential consequences of 65.)
So just to verify: a link to chart of implies for the target equation and all it's unknowns. I can put a PR up later tonight for that. What's a good name for that graph? https://teorth.github.io/equational_theories/graphiti/?render=true&implies=65,359,614,817,1426,1491,3862&highlight_red=65&highlight_blue=359,614,817,1426,1491,3862
I suppose what may also be nice is to have dashed edges between unknowns in the chart to also show what unknown relationships there are between the vertices, though maybe the unknown set is small enough now that that feature is no longer as useful.
Terence Tao (Oct 07 2024 at 17:34):
"Potential forward implications of EquationX"?
Similarly one can have
"Potential backward implications of EquationX" (proven + conjectured + open)
"Conjectured forward implications of EquationX" (proven + conjectured)
"Conjectured backwards implications of EquationX" (proven + conjectured)
similar to the current functionality of
"Proven forward implications of EquationX" (proven only)
"Proven backwards implications of EquationX" (proven only)
so maybe one just needs to add a dropdown feature next to the current "Equation implies" and "Equation implied by" text boxes to indicated whether implies/implied by means "proven only", "proven or conjectured", or "proven, conjectured, or open" (with the former being the default).
Terence Tao (Oct 07 2024 at 17:35):
One can also have options to include conjectural implications and open implications (dashed arrows and dotted arrows, perhaps?) within the visualization as you suggest, though turned off by default.
Terence Tao (Oct 07 2024 at 17:57):
Terence Tao said:
EDIT: the new system seems to be
If one takes a piecewise linear model
then (if my hand calculations are correct) the system becomes
and it should be possible to use a standard algebra package to see if this is solvable. (But it should be double checked, as one can see from past history I am making a lot of mistakes with this hand calculation.)
Daniel Weber (Oct 07 2024 at 18:01):
One thing to note is that the implication holds over finite models (as the magna is then left cancellative), so examples like this (which from what I understand imply that it has a counterexample in fields with large enough characteristic) can't work
Terence Tao (Oct 07 2024 at 18:10):
Ok... well one may have to go to noncommutative models then, where it should become possible to exclude finite models. The algebra should still be the same, but now one needs a noncommutative algebra package rather than a commutative algebra package to analyze it...
Terence Tao (Oct 07 2024 at 18:13):
This equation 65 is beginning to remind me of the village of Asterix and Obelix ("One small village of indomitable Gauls still holds out against the invaders...")
Daniel Weber (Oct 07 2024 at 18:24):
Daniel Weber said:
Terence Tao said:
Do you have proofs of these assertions written up somewhere? They might provide further clues.
[...]
Vampire proved them and I'm not at home right now, I'll send them in a couple of hours
The proof is via Equation 1491 x = (y ◇ x) ◇ (y ◇ (y ◇ x))
, which is immediate to deduce from left cancellativity and 65 by applying y
to the left
Daniel Weber (Oct 07 2024 at 18:25):
Terence Tao said:
From the diagram it seems we should test both the ring-theoretic and the function-theoretic constructions against 1491 first.
I see you mentioned 1491 earlier here, perhaps we should focus on 65 -> 1491
Terence Tao (Oct 07 2024 at 18:39):
Tellingly, 1491 is also the only equation whose implication into 65 remains open.
Zoltan A. Kocsis (Z.A.K.) (Oct 07 2024 at 21:28):
Daniel Weber said:
Could you explain the proof that the implication holds on finite magmas? I imagine that might guide searching for counterexamples
Sorry, I was traveling and mostly offline yesterday, just catching up with this thread. I see you've got the left-cancellability proof (it's the one I had, I've been a one-trick pony with my cancellative monoids in this project).
I picked 65 for good reason after your question about all remaining implications being false -
I've tried quite hard to construct infinte counterexamples after that, and bounced back hard. Glad to see in this thread that it wasn't just a "me" problem :sweat_smile:
Daniel Weber (Oct 08 2024 at 02:45):
Does equation 65 appear somewhere in the literature, by any chance?
Terence Tao (Oct 08 2024 at 02:55):
If it's not known, I (half-seriously) propose calling 65 "Asterix", and 1491 "Obelix".
Terence Tao (Oct 08 2024 at 04:27):
A simple observation: assuming 65, 1461 is in fact equivalent to left cancellability (since 1461 recovers x from y and yx). So the key question is whether models of 65 have to be left cancellative, ie left multiplication by y is injective. (Certainly it is surjective.)
Daniel Weber (Oct 08 2024 at 04:43):
Setting and quotienting by equation 65 it may be interesting to see what equivalence classes Vampire can prove, perhaps that could give some insight to how they look
Daniel Weber (Oct 08 2024 at 05:39):
Here are the (conjectured) non-trivial equivalence classes (where non-trivial means using equation 65). There's nothing interesting yet, but I'm doing a larger run now (which will likely take a few hours)
- : , ,
- : , , ,
- : , , ,
Hernan Ibarra (Oct 08 2024 at 06:39):
I think free semigroup on x,y modulo the equation (y x)^2 = x satisfies 65 but not 359
Hernan Ibarra (Oct 08 2024 at 06:40):
I don't have a proof of this yet (confluence might help; otherwise induction on the proof tree). Does it seem like it would work?
Daniel Weber (Oct 08 2024 at 06:41):
Sadly associativity + 65 implies 359, according to Vampire
Hernan Ibarra (Oct 08 2024 at 06:42):
Darn
Hernan Ibarra (Oct 08 2024 at 06:42):
Good to know though
Daniel Weber (Oct 08 2024 at 06:44):
In fact it even implies
Joachim Breitner (Oct 08 2024 at 06:44):
Is the rule (yx)(yx) -> x confluent, by a similar argument as 477? Probably not exactly the same argument, as it can apply on its own lhs's subterms, can it? But only if y = x, so maybe that helps with a (more complicated) confluence proof.
Daniel Weber (Oct 08 2024 at 06:45):
Daniel Weber said:
Here are the (conjectured) non-trivial equivalence classes (where non-trivial means using equation 65). There's nothing interesting yet, but I'm doing a larger run now (which will likely take a few hours)
[...]
This finished. Any patterns you can see here? (I don't include values which contain , as that's immediately reducible)
- : , ,
- : , ,
- : , ,
- : , , , , ,
- : , , , , , , , , , , ,
- : , , , , ,
- : , , , , ,
- : , , , , ,
- : , , , , ,
- : , , , , ,
- : , , , , ,
- :
- :
- :
- :
- :
- :
- :
- :
- :
Hernan Ibarra (Oct 08 2024 at 06:45):
Daniel Weber said:
In fact it even implies
Do you mind sharing the proof? I don't see it
Hernan Ibarra (Oct 08 2024 at 06:46):
Joachim Breitner said:
Is the rule (yx)(yx) -> x confluent, by a similar argument as 477? Probably not exactly the same argument, as it can apply on its own lhs's subterms, can it? But only if y = x, so maybe that helps with a (more complicated) confluence proof.
Yeah I thought it might be confluent for a similar reason but I haven't worked out the details yet
Joachim Breitner (Oct 08 2024 at 06:52):
Let's see. A term that can be rewritten in two (not independent) places has to be ((yx)(yx))((yx)(yx))
. So the critical pair consists of (xx)
if I apply the nested occurrences, and (yx)
if I rewrite on the outside. Doesn't look confluent to me, I fear.
Kevin Buzzard (Oct 08 2024 at 06:59):
Terence Tao said:
OK, trying again, this time with a general linear operation
x ◇ y = ax+by
. If I have calculated things correctly, Equation 65 becomes the systema(1+b^2)=0, b(a+b^2)=1
, and Equation 359 becomesa(a+b-1)=0
. Oh, interesting, here it does seem that again the former implies the latter. Ifa=0
this is clear, otherwise we have1+b^2=0
andb(a+b^2)=1
, and on multiplying the latter byb
and substitutingb^2=-1
we get after some algebraa+b-1=0
. OK, this explains why this wasn't picked up by the linear magma sweep.
This argument assumes that the base ring has no zero divisors ("if a=0
...otherwise we have 1+b^2=0
...") so it occurred to me that there was a little leeway here, but annoyingly even without this assumption the implication still holds:
import Mathlib.Tactic
example (R : Type) [CommRing R] (a b : R) (h1 : a * (1 + b * b) = 0)
(h2 : b * (a + b * b) = 1) : a * a + a * b = a := by
polyrith -- Try this: linear_combination (b ^ 2 + a - 1) * h1 - 1 * a * b * h2
Daniel Weber (Oct 08 2024 at 07:00):
Hernan Ibarra said:
Daniel Weber said:
In fact it even implies
Do you mind sharing the proof? I don't see it
Vampire found it:
By using equation 65 with , .
Now by equation 65 , so
Kevin Buzzard (Oct 08 2024 at 07:08):
Pace Nielsen said:
Using a map of the form x⋄y=ax+by+c, leads to the set of equations ba+b^3=1, a+b^2a=0, and a^2+ab\neq a. It turns out these are inconsistent over noncommutative rings. So no affine map with work over coefficients from a ring.
Oh in fact Pace was one step ahead of me :-) (although I only checked commutative rings)
Daniel Weber (Oct 08 2024 at 07:11):
together with 65 also implies 1491 :cry:
Daniel Weber (Oct 08 2024 at 08:59):
The equations that 65 doesn't imply, and together with it they still don't seem to imply 1491, are:
['Equation3076', 'Equation2053', 'Equation2054', 'Equation3078', 'Equation2567', 'Equation2060', 'Equation2063', 'Equation4629', 'Equation2584', 'Equation4121', 'Equation4636', 'Equation3105', 'Equation2088', 'Equation3115', 'Equation49', 'Equation2097', 'Equation2098', 'Equation4146', 'Equation4658', 'Equation4157', 'Equation4158', 'Equation4165', 'Equation3142', 'Equation73', 'Equation2125', 'Equation3667', 'Equation1109', 'Equation1112', 'Equation3675', 'Equation2660', 'Equation2670', 'Equation1648', 'Equation2672', 'Equation1654', 'Equation1655', 'Equation632', 'Equation1657', 'Equation124', 'Equation639', 'Equation2699', 'Equation2700', 'Equation1682', 'Equation1684', 'Equation1685', 'Equation2709', 'Equation669', 'Equation670', 'Equation159', 'Equation676', 'Equation677', 'Equation3749', 'Equation167', 'Equation679', 'Equation3752', 'Equation704', 'Equation1728', 'Equation706', 'Equation2243', 'Equation707', 'Equation4293', 'Equation3271', 'Equation713', 'Equation1229', 'Equation1231', 'Equation3279', 'Equation2263', 'Equation1241', 'Equation4321', 'Equation3308', 'Equation2804', 'Equation2293', 'Equation3318', 'Equation2300', 'Equation261', 'Equation1285', 'Equation263', 'Equation1288', 'Equation273', 'Equation3353', 'Equation2330', 'Equation1312', 'Equation2337', 'Equation1315', 'Equation2853', 'Equation2855', 'Equation1322', 'Equation1840', 'Equation2865', 'Equation2866', 'Equation819', 'Equation4405', 'Equation4406', 'Equation1848', 'Equation825', 'Equation1850', 'Equation2875', 'Equation2873', 'Equation833', 'Equation1860', 'Equation3925', 'Equation2902', 'Equation4442', 'Equation1885', 'Equation2910', 'Equation872', 'Equation1897', 'Equation879', 'Equation3952', 'Equation882', 'Equation2939', 'Equation4480', 'Equation385', 'Equation1922', 'Equation906', 'Equation907', 'Equation2447', 'Equation2449', 'Equation2450', 'Equation1428', 'Equation917', 'Equation3481', 'Equation1434', 'Equation2460', 'Equation1444', 'Equation1451', 'Equation429', 'Equation1454', 'Equation437', 'Equation3519', 'Equation1479', 'Equation1482', 'Equation2506', 'Equation1488', 'Equation1489', 'Equation466', 'Equation473', 'Equation476', 'Equation3548', 'Equation2531', 'Equation3555', 'Equation2533', 'Equation4071', 'Equation1518', 'Equation3056', 'Equation3058', 'Equation4083', 'Equation1526', 'Equation4599', 'Equation504', 'Equation3066', 'Equation2043', 'Equation3068', 'Equation3069', 'Equation4606', 'Equation511']
Will Sawin (Oct 08 2024 at 10:58):
Kevin Buzzard said:
Oh in fact Pace was one step ahead of me :-) (although I only checked commutative rings)
````
A tricky thing about commutative rings is any relation of the form "this equation holds but this one doesn't" that holds in a commutative rings with finitely many generators holds already in a happens for finite commutative rings (since these rings inject into the product of their finite quotients). So already knowing there are no finite counterexamples tells you you won't be able to make a counterexample with commutative algebra.
Terence Tao (Oct 08 2024 at 14:54):
Inspired by @Daniel Weber Vampire-driven exploration of the "Asterix" law 65 under the hypothesis 0 ◇ 1 = 0 ◇ 2
, I conducted by hand an exploration of the variant hypothesis 0 ◇ 0 = 0 ◇ 1 = 0
(with 0,1 distinct) and managed slightly more than half of an infinite multiplication table filled out. Not sure what to make of this, so I thought I'd record what I had here.
I'm going to write for the left-multiplication operators, so 65 becomes , and our hypothesis is that . If we define , then we have , thus (so in particular 2 is distinct from 0,1). If we then define , then , so (so in particular 3 is distinct from 0,1,2). Continuing in this fashion, we obtain distinct elements in the magma with
and for .
Next, we have , thus . Then , so . , so . By induction we see that whenever .
In a similar vein, , so ; , so ; and by induction whenever .
A further induction now tells us that when and , and we had also previously established when . That's about half of the multiplication table on (the upper-triangular region and one lower diagonal). I have had trouble filling in the rest of the table, though, which may be a good sign since perhaps these hypotheses are in fact contradictory.
Daniel Weber (Oct 08 2024 at 15:11):
Vampire can't find a contradiction to this
Daniel Weber (Oct 08 2024 at 15:14):
Looking at the quotient of the free magma by the rules you describe, Vampire found the following equivalence classes which aren't found by the multiplication table:
- : , , ,
- :
- :
Daniel Weber (Oct 08 2024 at 15:16):
What happens if you set all values not described by to 0? It seems to work here
Daniel Weber (Oct 08 2024 at 15:21):
No, then
Daniel Weber (Oct 08 2024 at 15:30):
I can try to fill values for the multiplication table with Vampire, each time setting it to the smallest value which doesn't let it derive a contradiction, and maybe it'd get stuck (which would mean we have to use values outside of ) or we'd spot a pattern
Zoltan A. Kocsis (Z.A.K.) (Oct 08 2024 at 15:35):
For the record, I tried a similar approach a couple of days ago without spotting a pattern. My issue was that I could go really quite far before reaching a contradiction even when I filled in the table in a commutative way. But we know that commutativity together with 65 implies left-cancellativity, so eventually continuing that particular table should become impossible. It just takes longer than my patience and computational capability extended.
Daniel Weber (Oct 08 2024 at 15:46):
It makes this
| * | 0 | 1 | 2 | 3 |
|---|---|---|---|---|
| 0 | 0 | 0 | 1 | 2 |
| 1 | 2 | 0 | 1 | 2 |
| 2 | 0 | 3 | 1 | 2 |
| 3 | 0 | stuck | none | none |
Terence Tao (Oct 08 2024 at 17:00):
Hmm, perhaps one has to extend the domain beyond the natural numbers then. Here is a possible "translation-invariant" ansatz. Let G
be an abelian AddGroup
, and consider a magma operation on G
of the form y ◇ x = x + f(x-y)
for some function f : G → G
. If I have computed correctly, Equation 65 then simplifies to the functional equation
f(h) + f(f(h)) + f(h + f(h) + f(f(h))) = 0
(*)
for all h : G
. Left-cancellability corresponds to the injectivity of h ↦ h + f(h)
. (This function is necessarily surjective, since it will map h + f(h) + f(f(h))
to h
thanks to (*).)
The partially filled multiplication table above corresponds to trying to work out f
on the integers, and getting as far as f(h) = -1
for h ≥ 0
and f(-1) = 2
. This verifies (*) for all h ≥ -1
. Not sure how to fill out the rest of f
though.
[EDIT: This so looks like an Olympiad problem. Time to ping Deepmind?]
Kevin Buzzard (Oct 08 2024 at 18:23):
I must confess that I spent some time two days ago pinging some ATP experts about this particular problem, but warned them that smart people had already been throwing some of their favourite toys at it. Clearly desperation is setting in! That comment above about "I wonder if it's independent of ZFC" is more evidence of this :-)
Thomas Browning (Oct 08 2024 at 18:33):
Perhaps I'm missing something, but if x ◇ y = x + f(x - y)
, then equation 65 seems to become
x = y ◇ (x ◇ (y ◇ x))
= y + f(y - (x ◇ (y ◇ x)))
= y + f(y - (x + f(x - (y ◇ x))))
= y + f(y - (x + f(x - (y + f(y - x))))
so
y - x + f(y - x - f(x - y - f(y - x))) = 0
or equivalently,
h + f(h - f(-h - f(h))) = 0
but I don't see how this relates to (*).
Terence Tao (Oct 08 2024 at 18:45):
So sorry! I had written x ◇ y
where I should have written y ◇ x
(it's the same ansatz, but represented differently; I've edited my previous post). The calculation is as follows: if x = y + h
, then
y ◇ x = x + f(h)
x ◇ (y ◇ x) = x + f(h) + f(f(h))
y ◇ (x ◇ (y ◇ x)) = x + f(h) + f(f(h)) + f(h+f(h)+f(f(h)))
and so equation 65 becomes
f(h) + f(f(h)) + f(h+f(h)+f(f(h))) = 0
.
Also we have y ◇ (y+h) = y + h + f(h)
so left-cancellability is equivalent to injectivity of h + f(h)
.
I experimented with some other ways to represent the ansatz, but this one leads to the simplest-looking equations as far as I can tell. Your version is equivalent; I think what you call f(h)
, I would call f(-h)-h
.
Joseph Myers (Oct 09 2024 at 00:50):
Terence Tao said:
Hmm, perhaps one has to extend the domain beyond the natural numbers then. Here is a possible "translation-invariant" ansatz. Let
G
be an abelianAddGroup
, and consider a magma operation onG
of the formy ◇ x = x + f(x-y)
for some functionf : G → G
. If I have computed correctly, Equation 65 then simplifies to the functional equation
f(h) + f(f(h)) + f(h + f(h) + f(f(h))) = 0
(*)for all
h : G
. Left-cancellability corresponds to the injectivity ofh ↦ h + f(h)
. (This function is necessarily surjective, since it will maph + f(h) + f(f(h))
toh
thanks to (*).)The partially filled multiplication table above corresponds to trying to work out
f
on the integers, and getting as far asf(h) = -1
forh ≥ 0
andf(-1) = 2
. This verifies (*) for allh ≥ -1
. Not sure how to fill out the rest off
though.[EDIT: This so looks like an Olympiad problem. Time to ping Deepmind?]
I don't think these values of f
can extend to the rest of the integers, though I haven't formalized my argument or spent very long checking it, so it shouldn't entirely be trusted to be correct (and there might be unnecessary pieces in it as well).
Say h < -1
. If f(h) = 1
then (*
) reduces to f(h) = 0
, contradiction. If f(h) = 0
then (*
) reduces to f(h-1) = 1
, contradiction. If f(h) = -1
then f(h+1) = -1
and repeating you end up with f(-1) = -1
, contradiction. And if f(h) = 2
then f(h+1) = -1
, contradiction. So f(h)
is not in the interval from -1
to 2
for any h < -1
. So either f(h) <= -2
or f(h) >= 3
; in the latter case, f(h + f(h) - 1) = 1 - f(h) <= -2
, so h + f(h) - 1 <= -2
, so h + f(h) <= -1
, which is also trivial when f(h) <= -2
. So f(h) + h <= -1
for all h < -1
. In particular, f(-2) <= 1
so f(-2) <= -2
.
Now consider the function t(x) = x + f(x)
discussed above, for which it was noted that t(h + f(h) + f(f(h))) = h
; replacing f(h) + f(f(h))
by t(f(h)) = t(t(h)-h)
, we have t(h + t(t(h) - h)) = h
for all h
. We had above that t(h) <= -1
for all h < -1
.
In this equation t(h + t(t(h) - h)) = h
, substitute h = x + t(t(x) - x)
so that t(h) = x
; we get t(x + t(t(x)-x) + t(-t(t(x)-x))) = x + t(t(x)-x)
. Take some x
such that f(x) = t(x)-x < -1
(we know that x = -2
has this property). Then t(t(x)-x) <= -1
, so -t(t(x)-x) >= 1
, so t(-t(t(x)-x)) = -t(t(x)-x) - 1
, so t(x - 1) = x + t(t(x)-x) <= x - 1
, so t(x - 1) - (x - 1) <= 0
. As t(x - 1) - (x - 1) = f(x - 1)
, it cannot be 0
or -1
, so f(x - 1) < -1
. Inductively, f(x) < -1
for all x < -1
. But then the LHS of (*) is negative for all such x, a contradiction.
Terence Tao (Oct 09 2024 at 01:28):
Huh, that's quite an intricate argument! The problem here is an immediate specialization of the "65 -> left cancellability" problem, so if this is the simplest proof available for this special case, then it strongly suggests that the general problem is also at least this complicated to prove. So perhaps it is worth trying to find a more streamlined proof. And the argument may be specific to one dimension (certainly the proof uses the total ordering of the integers quite a bit!); if one works with larger groups, e.g., Z^2, then maybe the equation becomes solvable again.
Will have to think about this more...
Daniel Weber (Oct 09 2024 at 03:33):
In the other direction (1491 -> 65), the question is whether has to be surjective (and because it has to be injective, that implication also holds in finite models)
Daniel Weber (Oct 09 2024 at 03:43):
This means that there's a function such that . Does completeness imply that if such an always exists then it's just an evaluation of some fixed term in the free magma over ?
Daniel Weber (Oct 09 2024 at 03:45):
Ah, never mind, works iff 1491 implies 65, so that's not interesting
Terence Tao (Oct 09 2024 at 03:50):
I don't think the completeness theorem can handle existential statements very well, it's just something special about 65 and 1491 that they relate to the surjectivity and injectivity of left-multipication somehow.
This is a very minor comment, but the original law 359 in this thread corresponds in the above model to . 1491 corresponds to something messier (if I computed correctly, it is but I am not 100% sure of this). This pair of equations (65 and 1491) are such weird equations: tantalisingly close to being understandable, but not connected as far as I can tell to any more standard mathematical structure...
Terence Tao (Oct 09 2024 at 08:03):
I think I was able to show that there are functions obeying the Asterix functional equation for which is not injective; this shows that indeed 65 does not imply 1491. The basic idea is to build the function greedily: every time one needs to decide what value has to be, select some number much larger than all previous numbers so that no collisions occur. It gets more technical than this because when one selects the value of at , one also has to select the value of at some related locations such as and , but this can be done by a somewhat technical induction. I wrote up the details at equational#453 and it should appear in the blueprint shortly.
The same method should also resolve the other anti-implications involving 65 or 1491. I'm going to sleep now, but tomorrow I can try to set out specific Lean formalization tasks to make this (somewhat complicated) proof completely verified (in this particular case this is important because there are a lot of fiddly details with the induction, even though the idea is broadly clear).
Daniel Weber (Oct 09 2024 at 09:42):
I'll start working on formalizing it
Daniel Weber (Oct 09 2024 at 10:33):
In Lemma 7.2, when you choose an element such that , and are all distinct and lie outside of , the finiteness of isn't enough, you also need . In the first case I understand how to get that, as you choose , but I'm not certain how to obtain that in the second and third cases.
Daniel Weber (Oct 09 2024 at 10:38):
I think adding the requirement that to the definition of a partial solution and requiring in Lemma 7.2 fixes it?
EDIT:
ah, but you can't get that in Corollary 7.4, in fact, necessarily.
What about setting and requiring for other values of ? I think that works, I'll try to continue with the formalization
Daniel Weber (Oct 09 2024 at 13:32):
Here's a slight simplification of Lemma 7.2:
The core operation is moving an element from to . This is the second part of the existing lemma, unchanged.
For an element we first add it to , by choosing some arbitrary and adding it to and setting . Then we move from to .
For an element it must be for some . We first move to and observe that this moved to , so we can now move it to .
Terence Tao (Oct 09 2024 at 14:21):
You're right, one should modify the notion of a partial solution by requiring and for all . Then one should modify the iteration a little bit to ensure the latter property propagates with the iteration.
As you note, one can seed the iteration with a situation in which and to get the iteration going, but one downside of that is that one only contradicts the Obelix equation and not the various single-variable equations downstream of that equation. However, I think one can seed the iteration also with a more complicated initial solution in which and things should still work (haven't checked this though).
I like your proposal to simplify the third case of Lemma 7.2 by first introducing a one-step version of the lemma.
I was initially thinking of breaking up the task of formalizing Section 7 into small pieces and distributing the proof out to different volunteers, but it sounds like you feel like you could do the entire thing, so I created a large task equational#463 to formalize the entirety of 65 !=> 1491 and also update the blueprint accordingly to implement the corrections and improvements you indicated above. If you would prefer to only perform a portion of the formalization / blueprint maintainance task, let me know and I will split the task into smaller pieces instead.
Terence Tao (Oct 09 2024 at 14:32):
I am optimistic that this method can also rule out the other unknown implications involving 65. I could set an explicit task for that as well, but perhaps the ongoing discussion here will resolve these organically? If you would like to informally claim one of these other tasks, you can "claim" it here and then I will set up a more official task in Github later.
Terence Tao (Oct 09 2024 at 14:58):
By the way, in case it helps, my conceptual model of the proof is that we are filling in the entries of f(h)
for various h
a few entries at a time, similar to solving a Sudoku puzzle; we are relying on the infinite nature of the puzzle to avoid getting "stuck". At any given point in the process, we will have a partially solved puzzle, with different type of numbers. The elements h
of are the "completely analyzed numbers": enough of the function has been determined that one can verify the Asterix functional equation for this choice of input h
. The elements h
of are the "partially analyzed numbers": we have f(h)
determined, but not enough of the rest of the function to resolve the Asterix equation here (but we have the capability to do so, by filling out a few more entries of the f
function table). The elements h
of are the "numbers of interest"; they have not yet had a value of f(h)
assigned to them, but have been selected as the output f(h')
of some other partially analyzed number h'
, and so are already slightly (but not excessively) constrained as to what values they can take. Everybody else in is an "uncontacted number" - this is an infinite pool of numbers that we can draw from to keep filling out our function.
The whole procedure reminds me of the technique of forcing in model theory, from what I have gathered about that technique over the years. I have had it on my "to do" list for some time to actually learn this technique; now I have some impetus to do so.
Pace Nielsen (Oct 09 2024 at 14:59):
This idea may be half-baked, but I thought I'd share it anyway.
Instead of restricting to be defined on , let's just define it on a general ring, and further assume it is linear . Then the Asterix functional equation becomes
Working in characteristic 3, this system works out to just say and . The map is not injective: both and map to zero.
By taking , and , we have a finite commutative ring. So this should give a finite counterexample (of size 81). (Hopefully I didn't make a silly mistake.)
Zoltan A. Kocsis (Z.A.K.) (Oct 09 2024 at 15:38):
We know that finite models of 65 are left-cancellative. Or am I misunderstanding what you're saying when you write that there should be a finite counterexample of size 81?
Will Sawin (Oct 09 2024 at 15:39):
The problem is that a^3 =a^2+a forces a to be invertible (the inverse is a^2-a-1) and so ab=0 implies b=0.
Will Sawin (Oct 09 2024 at 15:43):
I had a different idea related to defining f on a general abelian group. It seems the argument works without modification for an arbitrary countable abelian group. This suggests the following modification: Work on the free abelian group on infinitely many generators. Any time the argument asks us to pick an element outside some finite set, pick a new generator. Then we can label each generator by a label that expresses which step it was constructed on and which elements were used to construct it. Now it seems like the argument is producing some kind of free algebra with operations f, - and proving that various elements of the algebra are distinct. Then maybe it's possible to rephrase the argument in terms of the structure of the free algebra, without making choices, and maybe as proving some kind of confluence-like property?
Pace Nielsen (Oct 09 2024 at 15:45):
Will Sawin said:
The problem is that a^3 =a^2+a forces a to be invertible (the inverse is a^2-a-1) and so ab=0 implies b=0.
Not in a general ring. For instance, these equations are consistent with taking and .
Perhaps the issue with my argument is it doesn't force to be surjective. (And cannot, on pain of the problem you mention.)
Will Sawin (Oct 09 2024 at 15:56):
Pace Nielsen said:
Not in a general ring. For instance, these equations are consistent with taking and .
Oh sorry, that was silly of me. The problem is with the claim that both and map to , since maps to .
Daniel Weber (Oct 09 2024 at 16:18):
Will Sawin said:
I had a different idea related to defining f on a general abelian group. It seems the argument works without modification for an arbitrary countable abelian group.
You need to have coinfinitely many solutions for any , if you don't modify the argument (to find with )
Terence Tao (Oct 09 2024 at 16:30):
I certainly think we will need to figure out how to abstract this approach if we are to scale it to the hopefully dozens of other equations out there for which a similar method can apply. I agree with @Will Sawin that it does feel like some sort of "additive confluence" type of property, and that the free abelian group with countably many generators is actually the most natural domain to work in (in fact I had an early draft of the argument using exactly this group, but decided halfway to switch to the integers to make the proof look less scary from a notational perspective. [Actually I had an intermediate stage where I was working with a torsion-free infinite abelian group, with the torsion-free hypothesis needed to avoid the characteristic 2 issue @Daniel Weber just pointed out, but at that point I just decided that the integers were good enough.]
By the way if we do end up having a lengthy human-written proof of all the anti-implications involving Asterix and Oberlix, this would be a good test case for the duality metatheorems that we are making progress on formalizing in Lean, because I can imagine it would be a pain to manually dualize all of those human written proofs to settle the anti-implications involving dual-Asterix and dual-Oberlix.
Terence Tao (Oct 09 2024 at 17:20):
By the way, I wanted to note that the final (hopefully) working proof of the anti-implication 65->1491 was either directly or indirectly inspired by a lot of the previous discussion; definitely a collaborative effort, in the spirit of past Polymath projects!
For instance, @Daniel Weber 's Vampire explorations suggested that a collision in left-cancellability was only generating a very sparse set of additional relations, not enough to create a contradiction, so this hinted that one could "outrun" these relations on an infinite magma (and we knew early on that the magma had to be infinite). On the other hand, we had this partial solution on the integers which had the translation invariant structure that suggested the useful translation-invariant ansatz reducing things to a univariate functional equation; but as @Joseph Myers worked out, the infinite number of values that this partial solution already fixed made it impossible to complete the rest of the function. This helped give me the insight that one should only fix a finite number of values of the function at a time, so as not to run into these sorts of obstructions. Last, but not least, the negative results (by @Will Sawin, @Pace Nielsen , and others) showing that the ring-theoretic constructions were not working were important in order to allow me to finally let go of these ideas and pursue the more combinatorial approach that ended up being more fruitful.
So, a rather chaotic narrative with many twists and turns, but actually this is how many actual solutions of research-level problems happen - our published papers largely only describe (in a very polished fashion) the one approach that ended up working, but there are usually a half-dozen or more failed (or partially failing) approaches which preceded that approach, and in fact were essential to identifying and then implementing the one approach that could actuallywork.
Pace Nielsen (Oct 09 2024 at 19:04):
Thanks go to Will Sawin for finding my previous error.
Fortunately, I think the main idea can be salvaged and extended into a possibly workable automation scheme, as follows.
Instead of using a linear , make it quadratic, say (for simplicity) of the form . (The intuitive idea here is that it should be easier to make quadratics non-injective.) After some experimentation, it seems that working over a ring of characteristic makes things more workable. (Also, we may force and to commute, for convenience.) Then, if I didn't make any mistakes, we get a reduction system , , , and . To ruin injectivity we adjoin two more symbols where . Working out a reduction system, we get another five reductions , , , , and .
Since and are unaffected by these reductions, they are distinct. (Interestingly, if we make we are forced to get , so noncommutativity is quite important here.)
Terence Tao (Oct 09 2024 at 19:14):
I see. So basically you are using a quadratic ansatz to convert an intractable word problem to a ring reduction problem that might conceivably be proven to have good properties by existing methods from noncommutative ring theory (this is not my field (ha!), but it looks vaguely like you are implementing some noncommutative version of a Grobner basis?). It sounds like such counterexamples are going to be necessarily infinite, which is good as it gets around the objection that no counterexamples are possible in the finite setting.
Pace Nielsen (Oct 09 2024 at 19:16):
Terence Tao said:
I see. So basically you are using a quadratic ansatz to convert an intractable word problem to a ring reduction problem that might conceivably be proven to have good properties by existing methods from noncommutative ring theory (this is not my field (ha!), but it looks vaguely like you are implementing some noncommutative version of a Grobner basis?). It sounds like such counterexamples are going to be necessarily infinite, which is good as it gets around the objection that no counterexamples are possible in the finite setting.
Yes, that is exactly right. I'm using a noncommutative version of a Grobner basis computation (called the diamond lemma).
Will Sawin (Oct 09 2024 at 19:28):
Pace Nielsen said:
Thanks go to Will Sawin for finding my previous error.
Fortunately, I think the main idea can be salvaged and extended into a possibly workable automation scheme, as follows.
Instead of using a linear , make it quadratic, say (for simplicity) of the form . (The intuitive idea here is that it should be easier to make quadratics non-injective.) After some experimentation, it seems that working over a ring of characteristic makes things more workable. (Also, we may force and to commute, for convenience.) Then, if I didn't make any mistakes, we get a reduction system , , , and . To ruin injectivity we adjoin two more symbols where . Working out a reduction system, we get another five reductions , , , , and .
Since and are unaffected by these reductions, they are distinct. (Interestingly, if we make we are forced to get , so noncommutativity is quite important here.)
This is a great way to understand what is going on mathematically with this example. Since the equation 65 without left cancellability cannot hold in any magma that embeds into a product of finite magmas, this must be a noncommutative ring that fails to embed into a product of finite rings. Understanding what this ring is and why it fails to embed into finite rings in ring-theoretic terms could be a way to understand the theorem and why it's hard in more traditional mathematical terms.
Terence Tao (Oct 09 2024 at 19:29):
This may indeed scale better than my combinatorial approach, especially if one can leverage any existing software packages for noncommutative Grobner basis computations. Is there some source you can recommend to learn more about this topic? (Or would it be faster to simply write a new chapter of the blueprint with a very abridged introduction to the diamond lemma etc.).
Terence Tao (Oct 09 2024 at 19:30):
Presumably the moment one has a noncommutative polynomial map which is injective but not surjective, or vice versa, it stops being able to be embeddable into a product of finite rings.
Will Sawin (Oct 09 2024 at 19:30):
Are you assuming a and b commute with u and v here? It looks like all the expressions have a and b on the left and u and v on the right. In that case we can make use of the fact that the ring F_3[b]/(b^3-b^2-b) splits into a product of F_3[b]/b and F_3[b]/(b^2-b-1) to reduce to assume b satisfies one of these two equations. The first one implies a=0 so probably the second one is the interesting one.
Will Sawin (Oct 09 2024 at 19:32):
Terence Tao said:
Presumably the moment one has a noncommutative polynomial map which is injective but not surjective, or vice versa, it stops being able to be embeddable into a product of finite rings.
Not for injective but not surjective. For example the ring F_2[x] has the squaring map which is injective but not surjective but embeds fine into a product of finite rings. Surjective but not injective, this works.
Will Sawin (Oct 09 2024 at 19:34):
Maybe it's clearer to say that I'm hoping for an answer that relates this ring to known infinite-dimensional rings, e.g. to Heisenberg algebras or universal enveloping algebras of infinite-dimensional Lie algebras or something like that.
Terence Tao (Oct 09 2024 at 19:37):
One of my hopes for this project was to uncover "Mathematics from Mars": exotic objects that have comparable levels of rich structure as the textbook mathematical objects, but were overlooked by anything that did not resemble a systematic search, because they were largely disconnected from the tree of known mathematics. I don't know whether Asterix and Obelix are genuinely Martian mathematical objects, or are actually highly disguised versions of mathematical objects that are actually already known to terrestrial mathematics, but I am looking forward to finding out either way!
Pace Nielsen (Oct 09 2024 at 19:43):
Terence Tao said:
This may indeed scale better than my combinatorial approach, especially if one can leverage any existing software packages for noncommutative Grobner basis computations. Is there some source you can recommend to learn more about this topic? (Or would it be faster to simply write a new chapter of the blueprint with a very abridged introduction to the diamond lemma etc.).
George Bergman's paper here is the standard reference to the diamond lemma. Rather than have you wade through the details, here is the quick gist. To tell whether or not a sequence of reductions resolves to a normal form, you essentially just need two things. First, you need a well-ordering where all reductions result in linear combinations of smaller monomials in the ordering. (In practice, just use the length-lexicographical order.) Second, you need to check that overlaps resolve to a common expression. By an overlap, I mean that if we have two reductions like and , then the expression could be reduced in two different ways (according to where you place parentheses), and we get while . So we get a new relation . If all overlaps resolve, we have a system of reductions that yields a normal form.
I believe there are packages implementing this in Magma (and maybe others too).
Terence Tao (Oct 09 2024 at 19:44):
It's ironic that we haven't yet deployed Magma for this project
Terence Tao (Oct 09 2024 at 19:59):
I'm actually quite pleased to find out that there are two viable, but quite different, ways to analyze equation 65. We will hopefully be able to empirically start testing how well these two methods perform on the remaining unsolved implications. Will they have a comparable range of influence? Will one be better for one type of implication, and another better for a different type? This sort of experimental mathematics was another type of outcome I was hoping for with this project.
Will Sawin (Oct 09 2024 at 20:23):
Still assuming and commute with everything, saying the map fails to be injective is equivalent to the map so after changing the definition of it seems that it suffices to demonstrate the existence of an -algebra such that the map is not injective.
Will Sawin (Oct 09 2024 at 20:24):
Although I'm a little worried because doesn't that map have an inverse ?
Pace Nielsen (Oct 09 2024 at 21:08):
Will Sawin said:
Still assuming and commute with everything, saying the map fails to be injective is equivalent to the map so after changing the definition of it seems that it suffices to demonstrate the existence of an -algebra such that the map is not injective.
It turns out that if one makes u and v commute with a and b, then again the reduction system forces u=v.
Pace Nielsen (Oct 09 2024 at 21:09):
(deleted)
Will Sawin (Oct 09 2024 at 21:30):
Pace Nielsen said:
Will Sawin said:
Still assuming and commute with everything, saying the map fails to be injective is equivalent to the map so after changing the definition of it seems that it suffices to demonstrate the existence of an -algebra such that the map is not injective.
It turns out that if one makes u and v commute with a and b, then again the reduction system forces u=v.
So your calculations don't assume x commutes with a and b? Then why do all the formulas have a and b on the left?
Pace Nielsen (Oct 09 2024 at 21:34):
Arg, another error. Good point.
Will Sawin (Oct 09 2024 at 21:37):
One thing I observed is that if and are polynomials in a variable whose coefficients commute with and then since power series in with invertible constant term form a group under composition and hence left inverses are right inverses for them. So we can't use such polynomials for examples. But we don't assume the coefficients commute with , it's hard to check any identity between the polynomials since we'll have lots of terms with different variables inserted between copies of .
Pace Nielsen (Oct 10 2024 at 00:22):
Working over a commutative ring (so that evaluation of polynomials is a well-defined homomorphism!), I checked that if we take to be a quadratic polynomial solving the functional equation for Eqn65, then it also satisfies the functional equation for Eqn1491 (and vice versa). So no go here.
Terence Tao (Oct 10 2024 at 03:28):
Even if the noncommutative ring approach doesn't work for this particular equation, it's a good thing to keep in mind going forward. We still have 300 or so independent implications to resolve, and perhaps some of them will be amenable to this approach.
Daniel Weber (Oct 10 2024 at 10:26):
I finished formalizing Equation65_not_implies_Equation1491
successfully, now it just needs a bit of cleaning up
Daniel Weber (Oct 10 2024 at 10:27):
Should I try to make the resulting magma computable? That should be possible, but I'm not sure if it offers any benefits
Daniel Weber (Oct 10 2024 at 10:42):
I'll try to search for initial conditions to disprove all potential implications
Daniel Weber (Oct 10 2024 at 11:26):
I'm having trouble constructing partial solutions with :
Let's say we have . Then we must have .
Due to , this requires . Let .
Now we need , that is and . Because we must have , which requires
, so . Because then , this also implies , and we get
, which doesn't work because then , and isn't a bijection between and
Daniel Weber (Oct 10 2024 at 11:28):
Can the conditions be weakened to allow for ?
Pace Nielsen (Oct 10 2024 at 11:39):
Daniel Weber said:
Can the conditions be weakened to allow for ?
If I understand what you are asking for, then yes, the following should work. Take the direct product of Terry's combinatorial example that you formalized with the function in .
Daniel Weber (Oct 10 2024 at 12:03):
That works, but it isn't helpful for counterexamples as the part is always ok
Daniel Weber (Oct 10 2024 at 14:01):
Daniel Weber said:
Can the conditions be weakened to allow for ?
You need to add to , and then add to and you get , and then it has to be added to , and so on and so forth, so has to be infinite. This is a generalization of the earlier , which is stuck here, but perhaps in e.g. it can continue, by generalizing the finiteness of to some kind of thinness condition. I'll try that
Daniel Weber (Oct 10 2024 at 14:56):
I got that working, but that doesn't actually refute 359, for instance. It needs , which doesn't satisfy. Are there other such partial values of ?
Daniel Weber (Oct 10 2024 at 15:11):
Daniel Weber said:
I'm having trouble constructing partial solutions with :
Let's say we have . Then we must have .
Due to , this requires . Let .
Now we need , that is and . Because we must have , which requires
, so . Because then , this also implies , and we get
, which doesn't work because then , and isn't a bijection between and
In fact, this shows that Equation 65 implies Equation 359 in translation-invariant magmas, and I suspect all of the relevant one variable equations
lemma Equation65_implies_Equation359_ti (f : G → G) (h : @Equation65 G (translationInvariant f)) :
@Equation359 G (translationInvariant f) := by
rw [Equation65_translationInvariant_iff] at h
rw [Equation359_translationInvariant_iff]
have v1 := h 0
let h1 := f 0
let h2 := f h1
rw [zero_add, add_eq_zero_iff_eq_neg'] at v1
change f (h1 + h2) = -(h1 + h2) at v1
let h3 := f (-(h1 + h2))
have v2 := h (h1 + h2)
simp only [v1] at v2
convert_to -(h1 + h2) + h3 + f h3 = 0 at v2
· congr
abel
replace v2 : f h3 = h1 + h2 - h3 := by
rw [← sub_eq_zero]
convert v2 using 1
abel
have v3 : h3 + f h3 + f (_ + h3 + f h3) = 0 := h (-(h1 + h2))
rw[ v2] at v3
convert_to h1 + h2 + h1 = 0 at v3
· congr 1
abel
congr 1
abel
change h1 = f (- h1)
have v4 : -h1 = h1 + h2 := by
rw [eq_comm, ← sub_eq_zero]
trans h1 + h2 + h1
abel
exact v3
rw [v4, v1, ← v4]
abel
Daniel Weber (Oct 10 2024 at 15:14):
(deleted)
Terence Tao (Oct 10 2024 at 15:26):
Very interesting! So there is a limitation to the translation-invariant method. (Or, perhaps the 65 -> 359 implication is actually true!)
This is beginning to interact with the [recent disproof of 1661 -> 1657[(https://leanprover.zulipchat.com/#narrow/stream/458659-Equational/topic/1661.20-.3E.201657.20-.20another.20one.20bites.20the.20dust). In that construction, a "plain" translation-invariant magma did not work, but a finite modification of a (truncation of) the translation-invariant magma did work. I wonder to what extent the translation-invariant magma we constructed has the ability to be finitely modified, this could potentially be a way to resolve implications like 65->359 since 359 only has to fail at a single point.
Incidentally, upon reading up on the technique of forcing in model theory, I think the greedy algorithm used to construct the translation-invariant model is sort of a very simple version of forcing, which is about repeatedly adding "sufficiently generic" elements to one's model (in this case, a universe modeling ZFC) to achieve some specific law (one designed to have interesting consequences, e.g., the negation of the continuum hypothesis).
Daniel Weber (Oct 10 2024 at 15:29):
Could this induction be used directly to give values to the magma operation, without passing through translation-invariance?
Daniel Weber (Oct 10 2024 at 15:34):
For instance, say there are four right universes, . The operation is defined , we want and for . I don't know what additional conditions are needed or how to add/move values
Terence Tao (Oct 10 2024 at 15:46):
Wish I had time to think about this today, this sounds like an interesting approach! The one observation I had is that this type of construction will not contain the previous translation invariant construction as a special case, but will be a different (though analogous) construction. But perhaps that's what's needed here. On the other hand, the fact that the equation is now bivariate instead of univariate suggests to me that there will be a lot more "coupling" between different equations, and one cannot independently tweak the values of f
in some places without causing breakages in others, unless somehow one is very clever with how one sets up the induction (in particular, I wonder if one can even hope to make f
as "injective as possible", subject of course to the non-injectivity caused by 65, and the minimal amount of non-injectivity required to break other laws )
Daniel Weber (Oct 10 2024 at 16:03):
Perhaps the pairs can be categorized based on how much of y * (x * (y * x))
is defined?
Terence Tao (Oct 10 2024 at 16:35):
That sound promising (it looks compatible with the translation-invariant construction).
One might also try this approach with the specialization
of the problem introduced some days ago. The point here is that appear in these constraints relatively lightly, and so might be easily "forceable"; still appears a lot, but never three times in the same equation, and so maybe there is a bit more flexibility here.
Finally, it seems that your construction on , while it does obey 359, 1426, 4065, 614 actually contradicts 3862 and 817, if I computed correctly. So it does squeeze out two more anti-implications (and we get another two by duality).
Daniel Weber (Oct 11 2024 at 02:40):
Using could work there, perhaps? It gives , , and , and requires
Terence Tao (Oct 11 2024 at 02:57):
I'll play with this later this evening. Certainly it can't be worse (from a logical strength perspective) than the vanilla Asterix functional equation, since it contains that one as a special case when . On the other hand the previous obstruction that prevented looks like it might no longer apply here, so it looks promising.
Daniel Weber (Oct 11 2024 at 03:55):
I think I managed to get it to work directly on the magma:
We define a partial solution using two finite sets , and a magma operation . For any we want , , and . For any we want . Additionally, we want that for any such that , we also have and .
The main operation is adding a value to . We add a pair , setting to some which is different from all values mentioned in the partial solution (and ). We'll also add and set .
can't violate any condition, and the only way violates a condition is some having .
We will push all of these values to . That requires adding to and setting . Adding isn't problematic because , and isn't in the range of . The third condition is only relevant if , and then takes care of it.
The only potential problem remaining is if , which causes the pair to break . That means , and we have pushed it by setting . This lets us move to , as then
Terence Tao (Oct 11 2024 at 05:40):
Nice! In order to understand your argument, I rewrote it as follows. Define a shift map to be a function from to itself, such that the first coordinate of the output equals the second coordinate of the input. It is clear that such shift maps must take the form for some magma operation , giving a one-to-one correspondence between shift maps and magmas. We say that a shift map has the Asterix property if, whenever one has a chain of shifts (i.e., shifts to and shifts to ), then we also have . By unpacking the definitions, we see that a shift map has the Asterix property if and only if the corresponding magma operation obeys the Asterix law 65.
We make the following remark: if a shift map has the Asterix property, and shifts to , then must also shift to . Indeed, must shift to some , then by the Asterix property applied to , must shift to ; but then by the Asterix property applied to we obtain the claim. This remark helps motivate one of the conditions below.
To build shift maps, we define the notion of a partial shift map. This consists of two nested finite sets , and a shift map defined on . Let's call pairs in , , and "green", "yellow", and "red" respectively (this is to invoke the standard traffic light colors). We require the following axioms:
- If is yellow, then its shift must be red.
- If is green, then its shift is green or yellow, leading to a chain ; furthermore, is green or yellow, and shifts to .
- If is yellow and shifts to , then must also be yellow and shift to .
Now let be red. We would like to promote it to be either yellow or green. There are two cases.
CASE 1: It is not the case that is yellow and shifts to . Let be all the yellow pairs that shift to ( can be zero). We pick a new natural number not previously encountered, promote the to green, promote to yellow (with shift ), and promote the to yellow (with shift ). One checks that this preserves all the axioms.
CASE 2: is yellow and shifts to . This forces (since is red), and also that shifts to . Let the yellow pairs other than that shift to . We pick a new natural number , promote to green, to yellow (with shift ), and the to yellow (with shift ). One checks that this preserves all the axioms.
One can now promote any yellow pair to green, by promoting its (necessarily red) shift to either yellow or green by the above procedure, which will turn as a byproduct.
To contradict 359, start with a partial shift map in which is yellow and shifts to , is yellow and shifts to , and all other pairs are red. This can be checked to be a partial shift map, and corresponds to a magma where and , violating 359.
Daniel Weber (Oct 11 2024 at 12:54):
Should I add this proof to the blueprint? I finished the Lean formalization, equational#513
Daniel Weber (Oct 11 2024 at 13:19):
I wonder if this technique can be used to construct a model for equation 5105, perhaps just with translation invariance
Daniel Weber (Oct 11 2024 at 14:39):
I'll try to teach aesop
to do the relevant case analysis, that should let us apply this method to other problems without too much pain
Daniel Weber (Oct 12 2024 at 12:57):
Here's a general framework of these kinds of forcing arguments:
- We have a partial definition of the magma operation.
- We consider the set of all instantiation of variables in the law. At the start, these will all be unevaluated, and as we define values for the magma operation we will evaluate these in the equations. Whenever we get or in this set we will take it from this set and move it to the magma definition.
- Whenever we add a value to the definition, we set it to a fresh value , and we resolve this application to in all definitions.
- Now this is the tricky part: there might be definitions which now resolve to or , and we need to add them to the magma definition, resolve them in other places, and show it doesn't lead to contradictions.
- For equation 65, for example, this argument is: "suppose we're defining . If there was in the set of equations (i.e. ) we get , so we add all of these. If there was in the set of equations it will resolve to , which is reduced unless , as then we've added , and to fix this we add the requirement and define "
Daniel Weber (Oct 12 2024 at 14:34):
(deleted)
Terence Tao (Oct 12 2024 at 15:52):
Thanks for this explanation. Again, for my own understanding, I'm going to rephrase what you said in my own words.
We're basically trying to fill out a multiplication table on ℕ × ℕ
like solving a Sudoku puzzle. A partially defined magma is like a partially solved Sudoku puzzle. For any partial state there are some obvious "moves" one can do to fill in more entries, by substituting in the already solved values into the laws of the game. For instance, if the Sudoku rules consist only of the Asterix law x = y ◇ (x ◇ (y ◇ x))
, and one has already filled in 1 ◇ 2 = 3
and 2 ◇ 3 = 4
, then one must also fill in 1 ◇ 4 = 2
from the x=2, y=1
specialization of the Asterix law. Of course, if you have already filled in 1 ◇ 4
to equal some other value, then you have lost the game. But let us say that a partial magma is "locally complete" if all the obvious moves one could accomplish in this fashion were already in your partial solution. So, for instance, in a locally complete partial solution to the Asterix law, if the partial solution already asserts that 1 ◇ 2 = 3
and 2 ◇ 3 = 4
, then it must also assert that 1 ◇ 4 = 2
. (More generally, local completeness for the Asterix law is equivalent to the assertion that whenever y ◇ x = z
and x ◇ z = w
, then y ◇ w = x
.)
Let us say that a Sudoku ruleset (i.e., a set of laws, otherwise known as a "theory" in mathematical logic) is "greedily solvable" if, given any finite locally complete partial solution, and any relation a ◇ b
not yet defined by that partial solution, there is a way to extend that solution to a larger finite locally complete partial solution, in such a way that a ◇ b
is now defined. If we have this greedy solvability property, then a routine iteration (using some countable enumeration of ℕ × ℕ
) shows that any finite locally complete partial solution can be extended to a global solution of the given ruleset.
There is an obvious way to try to establish greedy solvability: set a ◇ b
equal to some natural number c
that is novel (not equal to a
or b
, or any number already appearing in the finite partial solution), and attempt to complete it under obvious moves. If one can always avoid a contradiction when doing so, one has greedy solvability, hence the extension property, and one can then use this to build many useful models of one's ruleset to create anti-implications.
So, let's try to see if the Asterix law x = y ◇ (x ◇ (y ◇ x))
is greedily solvable. Suppose we have some partial solution, and we now want to extend it by imposing a ◇ b = c
where c
is novel. There can now be some obvious moves: if the partial solution already has y ◇ a = b
for some y
, then the x=a, y=y
case of the Asterix law then forces y ◇ c = a
. That does not directly create any contradictions because c
is novel. However, if the partial solution has b ◇ a = b
, then this argument forces b ◇ c = a
, and then the x=b, y=a
case of the Asterix law forces a ◇ a = b
. This could lead to a contradiction if the partial solution already specified a ◇ a
to equal some other value. So unfortunately the Asterix law, by itself, is not greedily solvable.
However, we can fix this by adding a new law to prevent this scenario. So now our Sudoku rule set consists of two rules: the first is the Asterix law x = y ◇ (x ◇ (y ◇ x))
for all x,y
, and the second is the requirement that x ◇ x = y
whenever y ◇ x = y
. @Daniel Weber 's previous construction is then basically verifying that this rule set is greedily solvable: one can always add a new entry a ◇ b = c
to a finite locally complete partial solution with a novel c
. If one does not have b ◇ a = b
, one has to add y ◇ c = a
whenever y ◇ a = b
; if one does have b ◇ a = b
(and hence a ◇ a = b
, by hypothesis), one also has to add a ◇ c = a
and b ◇ c = a
(by the first rule) and hence c ◇ c = a
(by the second rule), and then a somewhat tedious check then verifies that one is now locally complete again.
I'll try later today to see if the laws 1076 and 73 that @Pace Nielsen resolved are also amenable to this technique. Another natural candidate is the Oberlix law 1491, since we still haven't resolved whether this implies the Asterix law. Hopefully this will shed some light on whether this process is automatable.
Daniel Weber (Oct 12 2024 at 16:11):
Here's a proof for 1491:
We will add two rules:
(1) if (y ◇ x) ◇ c = x
then y ◇ (y ◇ x)
is defined and equal to c
(2) x ↦ y ◇ x
is injective for any y
Suppose we're setting a ◇ b = c
, where c
is a new value. The equation b = (a ◇ b) ◇ (a ◇ (a ◇ b))
will reduce to (*) b = c ◇ (a ◇ c)
which is fine. If b = a ◇ x
(there is a unique such x
by (2)), there is also another equation x = (a ◇ x) ◇ (a ◇ (a ◇ x)) = b ◇ c
and we need to set (a ◇ x) ◇ c = b ◇ c = x
. This is OK with (1) by definition, and it's ok with (2) because if there was any (a ◇ x) ◇ d = x
then by (1) a ◇ (a ◇ x) = a ◇ b
would've been equal to d
, but we assumed it was undefined.
If a = b = a ◇ x
then (*) will further reduce to c ◇ x
, so we need to add c ◇ x = b
, which is ok with (2), and is ok with (1) because (a ◇ b) ◇ x = b
and a ◇ (a ◇ b) = a ◇ c = b ◇ c = x
Terence Tao (Oct 12 2024 at 16:30):
One might need a bit more analysis here. If for instance we already have b = a ◇ x
(so that we are forced to have x = b ◇ c
) and we also already have b ◇ x = y
for some y
, then 1491 forces c = (b ◇ c) ◇ (b ◇ (b ◇ c)) = x ◇ y
, so we have to add x ◇ y = c
into the mix as well. In particular there would be a problem if x ◇ y
were already set to some other value.
Daniel Weber (Oct 12 2024 at 16:39):
This represents the rule "if (a ◇ x) ◇ x = y
then x ◇ y
is equal to a ◇ (a ◇ x)
(and if one isn't defined so is the other)", right?
Terence Tao (Oct 12 2024 at 16:43):
Ah, okay, I see now, thanks.
So now I guess we just need to find a partial solution to the above ruleset that violates the Asterix law...
Daniel Weber (Oct 12 2024 at 16:49):
Terence Tao said:
Ah, okay, I see now, thanks.
So now I guess we just need to find a partial solution to the above ruleset that violates the Asterix law...
Adding this rule might not be enough, as setting x * y
will change more values, and it's possible that y = x * z
, and it can continue like this, so one has to check that this can't generate contradictions
Terence Tao (Oct 12 2024 at 16:53):
Well, we don't need to actually add the Asterix law to the ruleset. We could start with say 1 ◇ 0 = 2
, 0 ◇ 2 = 3
, and 1 ◇ 3 = 4
, which already violates Asterix (since 0 != 1 ◇ (0 ◇ (1 ◇ 0))
), and see if anything is forced from this and your ruleset (1), (2) (and perhaps one also needs to add Oberlix itself to the ruleset, as it isn't quite implied by (1), (2) as far as I can tell, being sort of a converse to (1)). From a cursory glance it seems that nothing is forced from this, and so it should be possible to extend this three-entry partial multiplication table to a complete solution to Oberlix that also violates Asterix.
[Side note: the most natural name for a model that obeys Oberlix, but does not obey Asterix, would be "Dogmatix".]
Daniel Weber (Oct 12 2024 at 17:00):
I meant that the rule "if (a ◇ x) ◇ x = y
then x ◇ y
is equal to a ◇ (a ◇ x)
" doesn't suffice to show that the multiplication table can be completed, as when using it you need to define x ◇ y = c
, which implies more stuff just like setting a ◇ b = c
previously did, and it's not obvious that this won't generate contradictions
Terence Tao (Oct 12 2024 at 17:26):
Ah, right, we need to revisit the analysis of your previous ruleset (1)+(2) to acccomodate the new rule, let's call it (3). (I had thought that (3) was just (1) in disguise but on closer inspection I see that it is a genuinely different rule.) If it doesn't close and it generates a lot more consistency conditions that then need to be added to the ruleset then this would indicate that this greedy approach is unlikely to be a good approach to construct Oberlix solutions.
Last updated: May 02 2025 at 03:31 UTC