Zulip Chat Archive
Stream: Equational
Topic: About 1729 vs 817
Shreyas Srinivas (Nov 11 2024 at 03:10):
So I don't have much time and I only got to work on this equation with z3 since the middle of this week. This list isn't complete even with what I have now. So far I have some rather trivial insights:
- Firstly I chose z3 because it had an easily accessible python API. I believe it is not too hard to adapt this to cvc5 since that one has a nearly identical python API.
- I have conducted most of my runs on
Int
s as the canonical infinite domain. - A few trivial things that I think are already known or easily visible by a quick glance at the equations: the binary operation of the Magma refuting the implication has to be : non-associative, non-commutative, non-idempotent. Further it cannot have a left identity.
- I have a conjecture based on experiments that restricting the range of values of or from above and below, within which they can deviate from the projection operations does not yield a counterexample. EDIT : z3 confirms this.
I will add more in the next few days to the above. In addition, and to a smaller extent, I have basically been trying to apply the methods of 1323 to this and none of the methods have yielded a counterexample so far. That being said, my goal there was to replicate the methods, and it was easiest to do so on finite examples and we don't expect finite counterexamples for this one.
Shreyas Srinivas (Nov 11 2024 at 03:11):
The reason I checked the last point is the way z3 was presenting its models of functions: A tabulation of values for small integers and a projection function for all other values.
Shreyas Srinivas (Nov 11 2024 at 03:13):
Point 4 above and some basic runs on z3 suggest to me that Integers (although SMT solvers have a great theory for them usually) are poor candidates for finding a counterexample. For instance, a few days ago z3 and cvc5 had a lot of trouble trying to find an operation satisfying 1729 (which is trivially satisfied by subtraction) without extra hints.
Shreyas Srinivas (Nov 11 2024 at 03:13):
Lastly, apologies for not getting to this earlier. I have been under extreme time constraints. Also, if any of this gets double posted, I am sorry about that too. Zulip's android app gives me a lot of trouble in this department
Terence Tao (Nov 11 2024 at 16:16):
Thanks for the update! I am suspecting that if one is to try to import the latest 1323-solving technology to 1729, one will need a good "base model" for 1729 on the squares, which would not directly refute 817, but could then be extended to non-squares. Looking forward to the full update!
Perhaps in the meantime, the following prepatory questions could be answered through ATPs, in analogy with how they laid the groundwork for the 1323 solution:
- Is it safe to assume that the 1729 model is unital? Does this lead to simpler formulations of the 1729 law?
- Is it safe to assume that the set of squares is closed under multiplication?
- Is it ruled out that the squares could be constant? What if the squares take only two values ?
Shreyas Srinivas (Nov 11 2024 at 16:31):
A small extension to the update : In my pen and paper work I wanted to find a natural way to create non-associative operations from simple ones. I came up with a "stateful operations" heuristic to do this. The idea comes to me from basic ML theory, where a larger hypothesis space is defined by parametrising over a smaller hypothesis space. (EDIT: In hindsight, it seems this can also be motivated by concurrency race conditions). The point is to have a bit more parametric control over the binary operation with the hope that SMT solvers have less trouble performing a parameter search than an uninterpreted function search for the full binary operation. All this is still a bit hazy and I want to run this on z3 and cvc5.
To give a trivial but illustrative example of this statefulness: Suppose the underlying domain is . Suppose is defined as where when and otherwise. Then whereas will be . The intuition here is that the state tracks the parity of number of operation uses and the use of non-associative operations in some cases ensures that the order of application of the individual instances makes a difference.
Shreyas Srinivas (Nov 11 2024 at 16:33):
Terence Tao said:
Thanks for the update! I am suspecting that if one is to try to import the latest 1323-solving technology to 1729, one will need a good "base model" for 1729 on the squares, which would not directly refute 817, but could then be extended to non-squares. Looking forward to the full update!
Perhaps in the meantime, the following prepatory questions could be answered through ATPs, in analogy with how they laid the groundwork for the 1323 solution:
- Is it safe to assume that the 1729 model is unital? Does this lead to simpler formulations of the 1729 law?
- Is it safe to assume that the set of squares is closed under multiplication?
- Is it ruled out that the squares could be constant? What if the squares take only two values ?
This sounds like a good starting point. I'll try these out
Terence Tao (Nov 11 2024 at 16:34):
This seems to align with some of the strategies we've tried successfully for other equations in which we assume there is a homomorphism from the desired magma to some small base magma (such as ) which often seems to clarify the algebra and enforce some good structural properties.
Shreyas Srinivas (Nov 11 2024 at 16:38):
Right, so I am approaching this from the point of view "What natural operations in computer science would not have the usual algebraic properties". It is trivial to find non-commutative operations (any monad would do). But non-associativity is much harder, since almost every nice data structure I can think of in CS has some sequential composition notion which corresponds to associativity. Things change when one adds statefulness
Shreyas Srinivas (Nov 11 2024 at 16:39):
and then the challenge is to start with basic non-associative operations and build more complex ones, and parametric ones.
Shreyas Srinivas (Nov 11 2024 at 17:15):
I think I ruled out the squares being +/-1 already, but I'll add an experiment to my notebook again to confirm this.
Shreyas Srinivas (Nov 11 2024 at 17:17):
Terence Tao said:
- Is it safe to assume that the 1729 model is unital? Does this lead to simpler formulations of the 1729 law?
Since I haven't been in a math dept for a while, I am guessing by unital you mean it has an identity element with left and right identity laws. The left identity law is ruled out. Having a right identity hasn't yielded much so far.
Shreyas Srinivas (Nov 11 2024 at 17:23):
basically 1729 is not consistent with a left identity rule
Shreyas Srinivas (Nov 11 2024 at 17:25):
Another observation, for the fallback conditions, when beyond a certain range of values of $x$, I implement subtraction as a fall back rule, even for large limits I get unsatisfiability. But when I turn the limit into a variable z3 can't find it. This wasn't the case when the fallback rules were projections
Shreyas Srinivas (Nov 11 2024 at 18:00):
The right identity law is also inconsistent with 1729
Terence Tao (Nov 11 2024 at 18:00):
OK, so imposing units is a bust. Good to know!
Shreyas Srinivas (Nov 11 2024 at 18:01):
I take that last one back. right identity is not confirmed yet. I had a minor error
Terence Tao (Nov 11 2024 at 18:04):
Another possible simplifying assumption is , i.e., squares are idempotent (equation 151), or for some constant (which will necessarily equal the right identity, if it exists).
Shreyas Srinivas (Nov 11 2024 at 18:05):
I already tried idempotence. I am currently on my machine and setting up everything in my notebook but not running any solver longer than 2 minutes.
Shreyas Srinivas (Nov 11 2024 at 18:05):
So far all the indeterminate runs have been run under 2 minutes.
Shreyas Srinivas (Nov 11 2024 at 18:12):
is ruled out for any constant
Shreyas Srinivas (Nov 11 2024 at 18:15):
Based on my experience so far, positive constraints narrow down the search much more quickly than negative constraints.
Shreyas Srinivas (Nov 11 2024 at 18:15):
at least positive equational constraints. This intuitively makes sense.
Terence Tao (Nov 11 2024 at 18:23):
Perhaps the most important remaining constraint to test is whether can be closed: the product of two squares is always a square. This seems rather key if one is to try a "build the multiplication table on the squares first" approach.
Shreyas Srinivas (Nov 11 2024 at 18:29):
Running it. I'll report back in a few hours.
Ted Hwa (Nov 11 2024 at 22:24):
Right identity is ruled out (assuming you are looking for a counterexample) since in equation 1729, , if 1 is a right identity, then substituting x=1 gives . Then equation 817 becomes which is true.
Shreyas Srinivas (Nov 11 2024 at 22:26):
That's my idea too but I want to coax z3 to say so
Shreyas Srinivas (Nov 11 2024 at 22:26):
In my earlier attempt I had forgotten to remove a different constraint which gave unsat
Shreyas Srinivas (Nov 11 2024 at 22:28):
Further attempts on left identity have shown too much variance in running times.
Shreyas Srinivas (Nov 11 2024 at 22:28):
And z3 didn't terminate the right identity for a long while
Ted Hwa (Nov 11 2024 at 22:34):
Vampire finds the proof for right identity instantly.
Shreyas Srinivas (Nov 11 2024 at 22:36):
Interesting. What's the ground theory you are using?
Shreyas Srinivas (Nov 11 2024 at 22:36):
Does vampire have some inbuilt support for equational reasoning that smt solvers don't?
Ted Hwa (Nov 11 2024 at 22:39):
I'm not familiar with internals of Vampire but I believe it does have support for equational reasoning, based on the proof it outputs.
Ted Hwa (Nov 11 2024 at 22:41):
The proof from Vampire is basically the same as the one I wrote above.
Shreyas Srinivas (Nov 11 2024 at 22:45):
Does vampire have an easy API in other languages
Shreyas Srinivas (Nov 11 2024 at 22:45):
So far I haven't seen anything in that direction. I will also try cvc5
Ted Hwa (Nov 11 2024 at 22:47):
It doesn't seem to have an API for other languages, only its own CLI interface
Shreyas Srinivas (Nov 11 2024 at 22:51):
Oh that's sad. I was hoping I could just plug it into a jupyter notebook. So far with z3 and a bit of cvc5, it has been very useful
Terence Tao (Nov 11 2024 at 23:49):
I suspect the 3-step procedure used to resolve 1516->255 has a good chance of working for 1729->817. The steps are:
- First build a 1516 model for the squares, with some additional properties TBD (analogous to the "double surjectivity" in the 1516 case) required to advance to step 2. In particular, the block of the multiplication table is now filled in: we understand "squares x squares".
- Work out the and blocks of the table ("squares x non-squares" and "non-squares x squares"). Here I think we mostly rely on the form of the 1729 law for . For squares, all the left and right multiplication operators are invertible, so for instance , which tells us that the "non-squares x squares" block of the table is determined by the "squares x non-squares" block. Some additional properties (analogous to the "infinite surjectivity" in the 1516 case) need to be imposed to advance to step 3.
- Fill in the last block of the multiplication table. This should be relatively straightforward because 1729 now reduces to a law of the form which looks easy to fill in greedily, assuming that we have had the foresight to implement some suitable "infinite surjectivity" type hypothesis in step 2.
Shreyas Srinivas (Nov 12 2024 at 00:02):
Ted Hwa said:
Right identity is ruled out (assuming you are looking for a counterexample) since in equation 1729, , if 1 is a right identity, then substituting x=1 gives . Then equation 817 becomes which is true.
Btw, to put it out there, this argument is important in my argument for left identity being inconsistent with 1729, since if there was a left identity, , using in 1729, it reduces to for every . Now this makes a right identity.
Shreyas Srinivas (Nov 12 2024 at 00:02):
Which in turn is inconsistent with negating 817
Shreyas Srinivas (Nov 12 2024 at 00:03):
One thing I must note is that z3 has been behind my mental math in almost all observations. The exception is the refutation of some fallback based operations.
Shreyas Srinivas (Nov 12 2024 at 00:05):
Terence Tao said:
I suspect the 3-step procedure used to resolve 1516->255 has a good chance of working for 1729->817. The steps are:
- First build a 1516 model for the squares, with some additional properties TBD (analogous to the "double surjectivity" in the 1516 case) required to advance to step 2. In particular, the block of the multiplication table is now filled in: we understand "squares x squares".
- Work out the and blocks of the table ("squares x non-squares" and "non-squares x squares"). Here I think we mostly rely on the form of the 1729 law for . For squares, all the left and right multiplication operators are invertible, so for instance , which tells us that the "non-squares x squares" block of the table is determined by the "squares x non-squares" block. Some additional properties (analogous to the "infinite surjectivity" in the 1516 case) need to be imposed to advance to step 3.
- Fill in the last block of the multiplication table. This should be relatively straightforward because 1729 now reduces to a law of the form which looks easy to fill in greedily, assuming that we have had the foresight to implement some suitable "infinite surjectivity" type hypothesis in step 2.
Sounds like a plan, although I should probably do this tomorrow. It is rather late now in my part of the world.
Shreyas Srinivas (Nov 12 2024 at 00:06):
It is possible I need to tweak/improve my way of using these SMT solvers, as the same heuristics don't seem to translate one-one to other ATPs
Shreyas Srinivas (Nov 12 2024 at 16:02):
I have been doing some not yet successful pen and paper work building off my "stateful operation" heuristic. At first glance this heuristic appears to allow us to have heterogeneous operations whose effect depends on the position of the operator's occurrence in the abstract syntax tree (AST) of an expression. For instance if one looks at the height of the operators in equations 817 and 1729. Let's use subtraction as our basic operation. Looking at the ASTs of 817 and 1729, it is clear that if we apply flipped subtraction () at height 3 nodes, we can break 817 and we can fix this breakage in 1729 by using flipped subtraction in height 1 nodes. For height 0 nodes we use normal subtraction.
However this is not enough. We homogenise these heterogeneous operations by encoding some extra data in the operands (for example by adding a height modulo 3 parameter to the domain) that carries some info about the . The operation itself needs to be defined uniformly on inputs regardless of the input height parameter. In particular 1729 must be satisfied independent of the height parameter component of the input arguments to the parameters and . nFor example a user might give an equation in which 1729's rhs is a subterm whose root occurs at height 5. It might receive as input values with varying heights. The goal is to get a better operation that is uniform w.r.t. input "heights"
Shreyas Srinivas (Nov 12 2024 at 16:10):
Maybe height of the operand node is the wrong parameter to focus on, although it seems easiest.
Jose Brox (Nov 12 2024 at 18:37):
Terence Tao ha dicho:
- Is it ruled out that the squares could be constant? What if the squares take only two values +1,−1?
Only two squares is quickly ruled out by Vampire-SAT (as expected, Prover9 is still running on it after 8 minutes...).
Terence Tao (Nov 12 2024 at 18:43):
@Shreyas Srinivas does it look like your stateful operation constructions could at least produce interesting infinite models of 1729 even if they cannot fulfill 817? They may be useful recipes for step 1 of the three-step procedure I mentioned previously.
If we wanted to pursue the 3-step strategy more, I think the first thing to do is focus on step 3: assuming that the multiplication table is already filled in , what axioms need to be satisfied on that portion of the table in order to be able to easily fill in the non-square portion by a greedy algorithm? Note that 817 doesn't directly care about this portion, as it can be tested purely using the component, so if we can get a clean criterion for solvability of the completion problem of the multiplication table from to , then this should resolve Step 3 and leave us just with working out the other two steps.
Shreyas Srinivas (Nov 12 2024 at 18:51):
With my model refuting 817 is easy. It is satisfying 1729 that is more difficult
Shreyas Srinivas (Nov 12 2024 at 18:52):
Because whatever extra parameters I tack on to integers, 1729 must be satisfied for all possible instantiations
Shreyas Srinivas (Nov 12 2024 at 18:56):
Basically the only structurally asymmetric occurrence of the operator in 817 is the first instance from the left (or the root of the AST). The modification of this occurence must be compensated for in 1729. In my example above, when using subtraction as a building block, this means flipping the height 2 occurrences
Shreyas Srinivas (Nov 12 2024 at 18:57):
But satisfying 1729 by itself without worrying about 817 is easy
Shreyas Srinivas (Nov 12 2024 at 18:57):
Subtraction satisfies it
Shreyas Srinivas (Nov 12 2024 at 18:57):
It's just not super useful
Shreyas Srinivas (Nov 12 2024 at 19:02):
Jose Brox said:
Terence Tao ha dicho:
- Is it ruled out that the squares could be constant? What if the squares take only two values +1,−1?
Only two squares is quickly ruled out by Vampire-SAT (as expected, Prover9 is still running on it after 8 minutes...).
I am really curious as to why vampire seems to be so much more successful than basically any other prover (including in several cases, just pen and paper work).
Terence Tao (Nov 12 2024 at 20:56):
Are you able to construct a model of 1729 in which the iterated squaring map is non-constant, where (so )? I have an idea on how to make the 3-step program work, but it requires a seed model in which is non-constant (more precisely I need the set to vary in a non-trivial way in , but presumably making non-constant will do this).
Shreyas Srinivas (Nov 12 2024 at 21:02):
Not yet, but I think there might be a way to do that on pen and paper. Intuitively, I just need to keep track of the number of continuous applications of an element to itself
Shreyas Srinivas (Nov 12 2024 at 21:03):
And reset the counter on non-contiguous occurrences, and also an extra state variable to keep track of the last value assigned to a cube
Shreyas Srinivas (Nov 12 2024 at 21:04):
Also keep the starting values of the counters in memory for reference. At this point I am just defining a Moore machine
Shreyas Srinivas (Nov 12 2024 at 21:07):
Sorry a mealy machine and then convert it to a moore machine.
Shreyas Srinivas (Nov 12 2024 at 21:07):
And then encode its table in an operator.
Shreyas Srinivas (Nov 12 2024 at 21:09):
I'll get on with this and report back in a few hours
Terence Tao (Nov 12 2024 at 22:02):
Actually I think I may just need a model with non-constant (not ).
The model I have in mind is that of an infinite submagma of squares (in which is non-constant, so will be non-constant in the entire magma), and then a larger set of non-squares , where and is in the free abelian group of exponent 2 generated by a generator of order 2 for each . The squaring map on non-squares is to be given by , and the left-multiplication by squares given by
These operators commute and are involutions, so the Ramanujan law then tells us what the right-multiplication by squares given by
If the squaring map is non-trivial enough, one should have take different values as varies. To get a 817 violation we need something like being non-trivial globally, so should be non-trivial on the submagma .
To fill out the remainder of the multiplication table for non-squares, there is a constraint , and 1729 for non-squares basically reduces to the law
This law iterates to produce 6-cycles similar to the 1323 construction, so I think there is a good chance of filling out the table by a greedy construction.
Shreyas Srinivas (Nov 13 2024 at 02:35):
I will need a bit more time. But I have had many false starts on the domain where the latter set has the usual order but increment and decrement, and consequently addition and subtraction wrap around (basically all operations on the second element are modulo 3). Intuitively, when the absolute value of height difference (denoted by 0,1,2). The base operation is subtraction of reals. To satisfy 1729, one must encoded that if the height difference on the left and right are 0 then apply normal subtraction whereas when they are not, apply flipped subtraction.
An alternative is that at 0 height difference apply flipped subtraction, at height diff 1, apply addition, and at height difference 2 apply normal subtraction. This can get a non constant square operation. The challenge is to figure out the correct formulation for the new height of the result of the operation. This has been my last few hours of work. At times it has taken me tantalising close to an answer only for me to find out that for each height assignment I have constructed so far, EQ 1729 breaks at some place or the other
Shreyas Srinivas (Nov 13 2024 at 02:43):
Breaking 817 is easy. So far I have been exploiting the only asymmetry in 817 which is the height 2 occurrence of , and I am using it as a guideline for constructing the conditional statement for switching operations.
Shreyas Srinivas (Nov 14 2024 at 16:29):
I am a bit tied up for the next 3 days. I'll post an update on Sunday. Hopefully I have a way to safely handle bad state inputs by then
Shreyas Srinivas (Nov 14 2024 at 16:30):
In the meantime, when I have a half an hour here or there to spare, I will try to post some of the simple examples as lean code here, so that others can modify and play with the idea.
Terence Tao (Nov 17 2024 at 04:08):
If constructing a base model is too hard, it may be possible to pull off a "swindle" and perform an infinite number of extensions to get a non-trivial model, without ever having to verify the base model properties at all, by pushing the base model further and further back in "time" and passing to the limit. I haven't really thought this idea through, but I guess we'll see first how the efforts to build non-trivial 1729 models are going.
Matthew Bolan (Nov 17 2024 at 04:15):
Did the recent correction to the argument for 1323 impact the idea to build a 1729 -> 817 counterexample from a model with non-constant?
Terence Tao (Nov 17 2024 at 04:20):
I think 817 has a different flavor to 2744, it only needs the "non-squares x squares" portion of the multiplication table rather than the "non-squares x non-squares" to refute. But I haven't worked out any details yet.
Terence Tao (Nov 17 2024 at 17:30):
Here is a negative result: if one has , then 817 holds. So this actually rules out the type of models used for 1323, as they obey this rule (at least for non-squares, in fact the model obeys the stronger law for non-square ); we need to find a more complex model that avoids this rule.
Proof: 1729 states that . Setting we obtain . Next, replacing by we have , so by invertibility of . Replacing by and using the hypothesis we have , hence . By invertibility of we conclude , but this is 817.
Conversely, 817, which is , clearly implies . So it is really the law that needs to be refuted, rather than .
Terence Tao (Nov 17 2024 at 19:11):
It may be useful to repeat the ATP-assisted exercise we have done in similar equations of trying to find additional axioms we can place on top of 1729 that can simplify the algebra without accidentally proving 817. So for instance would be an example of an axiom that we cannot impose; the laws and similarly cannot be imposed (the former implies the latter since ).
Terence Tao (Nov 17 2024 at 19:13):
Another observation: the identity just proven shows that the law 817 holds whenever is injective, in particular 817 holds for squares.
Shreyas Srinivas (Nov 17 2024 at 19:54):
I will have time to do this tomorrow. I'll try to run multiple ATPs
Terence Tao (Nov 17 2024 at 20:26):
Thanks! Some sample questions that ATPs may be able to answer (with partial confidence):
- Can we assume that squares are closed under multiplication, i.e., that for all there exists such that ?
- Can we assume there a right unit ? What about a left unit (which I think is stronger)?
- Can we assume is a constant? (Probably not.) What about ? Or maybe or could be viable axioms.
- Could left-multiplication by squares be abelian, thus ? This would also imply that right multiplication on squares is abelian. Separately, could we assume that left-multiplication by squares is an involution, ?
Shreyas Srinivas (Nov 19 2024 at 02:03):
Infinitesimal update: many z3 runs ongoing. I think I already ruled out being constant because in 817, would become an identity element, and our elusive counterexample can have neither left nor right identity
Shreyas Srinivas (Nov 19 2024 at 02:05):
Further, higher up in the thread we already have proofs that we can't have a right or left identity (one follows from the other)
Shreyas Srinivas (Nov 19 2024 at 02:33):
I think I am going to add to my list the following check: whether I can satisfy the one variable variant of 1729
Shreyas Srinivas (Nov 19 2024 at 02:33):
It won't be a valid counter example, but it might prune the search a bit
Shreyas Srinivas (Nov 19 2024 at 02:47):
My editor crashed with the square closure run (I am running z3 inside vscode)
Shreyas Srinivas (Nov 19 2024 at 02:54):
If is a constant, then even square elements cannot have a right identity (substituting in 817)
Shreyas Srinivas (Nov 19 2024 at 03:10):
left multiplication being involutive is consistent with 1729, but does not imply it fully. It doesn't seem inconsistent with 817
Terence Tao (Nov 19 2024 at 19:01):
Just reporting what would be needed to extend a base 1729 magma (representing "squares") to a larger magma (with representing "nonsquares"), thus we are restricting attention to models where the set of squares is closed under multiplication, and is already given to us somehow.
I will consistently use for elements of and for elements of (or ). This requires introducing a squaring map and to complete the original mutiplication table to . From the bijective nature of for we know that these maps have to permute the non-squares, thus we have to define bijections as well as the multiplication operation for non-squares.
1729 asserts that . For squares , we can rearrange this as
Thus the right-multiplication operators , are completely determined by the left-multiplication operators , .
Applying 1729 with and , we obtain , which we can rearrange as
This fills out part of the multiplication table on . One has to ensure that this rule does not collide with itself, or with the consistency condition
so we need the to be distinct from each other and from as varies (an exception can be made if , but we do not want to make this exception for all as this would precisely give 817).
1729 can also be written as
Applying this with (3) and we obtain the constraint
so is either a fixed point or a 2-periodic point of the permutation . Applying this instead with (2),we obtain
for and . We can change variables a bit and write this constraint as
It was tempting to simplify this law by asking that right-multiplication did not affect squares, so that . But then (5) and (4), together with the invertibility of , would simplify to
and setting we would obtain
which is 817. So we need right-multiplication to affect squares at least once .
Anyway, I believe (1), (4), (5) are the main constraints. If we can find a base 1729 magma and left and right multiplication operators for obeying (1), (4), (5) but not (817), and with the distinct from each other and from as varies, then we should be able to greedily fill in the rest of the table (providing is infinite and nothing too bad happens with the iteration).
Terence Tao (Nov 19 2024 at 21:39):
For the record, we have the following non-trivial model of 1729, which unfortunately obeys 817, but could potentially be a base model for a larger 1729 magma that violates 817.
Let be a countably infinite abelian group of exponent 2. The carrier is . The multiplication law is partially given by
So in particular . For the remaining products with distinct, these should be set to for some distinct from subject to the rule
This is a 6-periodic rule and can be filled out by the usual greedy algorithm.
It is not difficult to check that this obeys 1729. Unfortunately it also obeys 817: and for all . But perhaps we can use it as a base for a more sophisticated model.
If is a boolean algebra, we can in fact choose the explicit form
which I think was also observed in the 1323 thread by @Bruno Le Floch .
Shreyas Srinivas (Nov 19 2024 at 21:46):
If is a Boolean algebra, this operation is commutative
Shreyas Srinivas (Nov 19 2024 at 21:47):
So we have a lot to undo if we start there
Terence Tao (Nov 19 2024 at 21:50):
I am thinking of using this as a model just for the squares. If ATPs do not rule out the possibility of the squares being commutative, closed under multiplication, and unital, then having a boolean model for the squares may be viable.
Terence Tao (Nov 19 2024 at 21:52):
The squares would also obey , so the general magma would obey , but to my knowledge this has not been ruled out. (Also, is only a unit within the squares; it is not required to be a unit in the larger magma, and probably we would have to abandon that property.)
Terence Tao (Nov 19 2024 at 23:11):
Hmm, but I see from your previous post that one cannot have and a unit for the squares, so indeed the boolean model cannot serve as a base model. (But it could perhaps be a base for a base...)
Terence Tao (Nov 19 2024 at 23:30):
Hmm maybe you can clarify actually: if and is (say) a right unit for the squares, were you able to show that this implies 817 for all elements, or only for the squares? For if it is just the latter, we could still hope to use the boolean model as the base model to produce at least one contradiction to 817 (we don't need to contradict it everywhere, and I think in fact it automatically holds for squares in any case).
Terence Tao (Nov 19 2024 at 23:53):
The boolean example is also an abelian group of exponent 4, and conversely addition on any abelian group of order 4 is a 1729 magma (funny how I never noticed that before).
Shreyas Srinivas (Nov 20 2024 at 00:00):
So far I have not refuted identity elements on either side for only squares, only that they must exist
Shreyas Srinivas (Nov 20 2024 at 00:01):
The square closure is giving my z3 installation quite a bit of trouble
Shreyas Srinivas (Nov 20 2024 at 00:01):
It could just be that I am using an underpowered machine/software setup
Shreyas Srinivas (Nov 20 2024 at 00:03):
means that all square elements must satisfy 817 trivially.
Terence Tao (Nov 20 2024 at 00:12):
In fact I believe 817 holds for squares (i.e. ) even without any additional axioms beyond 1729, because we have , hence , hence .
Shreyas Srinivas (Nov 20 2024 at 00:55):
I don't quite see it right away. In the first step you have multiplied both sides of 817 by x.
Shreyas Srinivas (Nov 20 2024 at 00:55):
Where is 1729 used?
Shreyas Srinivas (Nov 20 2024 at 01:00):
(deleted)
Shreyas Srinivas (Nov 20 2024 at 01:09):
I am not sure we are thinking in the right direction with squares, because in squares + identity elements, we again find both 817 and 1729 satisfied, but it seems impossible to find a magma where non square elements also satisfy 1729 and not 817.
Shreyas Srinivas (Nov 20 2024 at 01:10):
But that's just going back to square one.
Shreyas Srinivas (Nov 20 2024 at 01:10):
The square conditions must surely be extraneous
Terence Tao (Nov 20 2024 at 03:28):
Shreyas Srinivas said:
Where is 1729 used?
Sorry, I was being brief (repeating arguments from earlier in the thread). The argument is as follows:
From 1729 one has , which we can rearrange as . Since is invertible, we conclude . If is a square , then is also invertible, so we conclude that 817 () holds for square numbers, or equivalently that for all .
Terence Tao (Nov 20 2024 at 07:40):
Here is an annoying obstruction:
Theorem. Suppose that a 1729 magma is such that is finite and closed under multiplication. Then 817 holds.
So we will need an infinite base magma if one is to try to build the counterexample starting from the squares.
Proof. Let ; our aim is to show that . For , we have by 1729, hence . So, if we set , it suffices to show that .
For any , we have
This already shows that the map is injective from to (since by hypothesis is injective and the bijection preserves the finite set ), hence is also a bijection. In particular there exists with , hence by injectivity of . Inserting this back into (1) we obtain , hence as required.
Terence Tao (Nov 21 2024 at 03:46):
I think I was finally able to get a greedy construction to work to refute 1729 => 817. The details are en route to the blueprint at equational#866 (EDIT: now landed), but the ideas are as follows.
- The carrier will be the disjoint union of a set of squares and a set of non-squares.
- For the squares , I took an infinite abelian group of exponent 4, which already obeys 1729. Because of previous obstructions, this was the simplest choice for that was available.
- Next, we select the right multiplication operators for . (It took me a while to realize that this was the component that had to be pinned down first, after fixing ; I spent way too long trying to pin down first.) Here I took the "free" option in which is the free non-abelian group generated by and is left-multiplication by . So there are no relations between any of the .
- Because of the 1729 identity for , we can write all the left-multiplication operators in terms of : indeed after some algebra one finds that (where by abuse of notation denotes left multiplication by ).
- One now has to select a map , a squaring map , and a multiplication operation obeying a certain number of technical axioms. It turns out that these axioms can be simultaneously satisfied by greedily selecting for together (I had previously tried to select each separately, but they were coupled together too annoyingly to do so).
There are two technical issues that complicate this greedy analysis beyond that of previous constructions. The first is that the 1729 identity implies that . As a consequence, every time one greedily selects , one is forced to also select an infinite number of additional identities and . But this is a relatively orderly injection of additional identities, and while annoying, does not cause major difficulties.
More tricky is dealing with the implication
that is a rephrasing of 1729, and which means that every time one fills in one entry of the multiplication table, another one also must be entered. In previous constructions there was a periodicity that let one terminate this iteration after a finite number of steps (six, in fact); but now that is constructed in a complicated fashion, and itself was also being constructed concurrently with the other data for the magma, I did not see a way to enforce this periodicity. Instead, I had to introduce a new category to the greedy construction, that of a "pending identity" such as , which we want to be true, but cannot yet implement because is undefined. So each time a new entry of the multiplication table is defined, one often has to place an identity such as on the "pending" queue, and later when is defined, any relevant pending identities on the queue then have to be incorporated into the multiplication table (which often then causes further pending identities to go on the queue). It's a bit convoluted, but I did not see a better way to achieve this.
Shreyas Srinivas (Nov 21 2024 at 13:48):
Awesome!! We still want to pursue a more "human-readable" counter-example right?
Shreyas Srinivas (Nov 21 2024 at 14:52):
@Mauricio Collares : I am referring to the second paragraph of the daily log of Day 47
Terence Tao (Nov 21 2024 at 15:44):
Certainly simpler constructions are always welcome! In particular they may be easier to formalize. I opened equational#869 to formalize the above argument, but if a simpler construction comes along it would make sense to formalize that instead.
That said, the large number of immunities this implication had suggests that any other construction may be difficult. I already found it challenging to create examples of a 1729 magma in which was not constant, for instance (probably I could do it by iterating the above construction, but I was not able to construct an algebraically simple example).
Matthew Bolan (Nov 21 2024 at 15:51):
I thought we knew linear models with that property, for example this one
Terence Tao (Nov 21 2024 at 16:50):
Oh, fair enough. I meant to say a model where was not surjective, and the iterates didn't stabilize until at least the third power . Though for the particular greedy construction I used, this wouldn't have been an obviously superior base model anyway, the point was it was hard to sustain genuinely non-surjective squaring over more than two iterations.
Kevin Buzzard (Nov 22 2024 at 06:41):
So you're now "mathematician-finished" but my instinct is not to celebrate until you're "lean-finished", because there may still be a twist in the story :-) Although it might be tedious to formalise the 80(?) or so "conjectures" we all know from experience that people can make mistakes... This is the "perspiration" after the "inspiration" in the old saying.
Congratulations to all, by the way! It's definitely a great milestone in the project.
Matthew Bolan (Nov 22 2024 at 06:56):
52 conjectures remain to be formalized, stemming from 13 or 14 equations.
Shreyas Srinivas (Nov 23 2024 at 02:57):
some of these appear non trivial to formalise so I'd say the field is still open for finding simpler counterexamples
Kevin Buzzard (Nov 23 2024 at 08:51):
Or for finding errors :-)
Last updated: May 02 2025 at 03:31 UTC