Zulip Chat Archive
Stream: new members
Topic: Any ideas for a formalization project?
Benoît Guillemet (Jan 25 2024 at 14:36):
Hello, I am a student in my first year of a master's degree in mathematics at ENS Paris-Saclay, France. Some friends and I would like to work on a small formalization project in Lean. Thus, we are searching for a theorem to formalize that is understandable at our level and that is not in Mathlib for the moment (so that our work might be useful).
Our areas of interest are geometry, algebraic topology, and category theory. We could also formalize a result in combinatorics, graph theory, or logic.
Does anyone have any ideas?
Kevin Buzzard (Jan 25 2024 at 14:52):
Singular homology!
Kevin Buzzard (Jan 25 2024 at 14:52):
The definition we use is quite "category-theoretic", and there is plenty of low-hanging fruit (like singular homology of basic spaces such as n-space or the n-sphere). Better check amongst the experts that this is not yet (a) done or (b) being worked on, but I am pretty sure that we're ready for it and it would be very cool to have it.
Kevin Buzzard (Jan 25 2024 at 14:55):
here is Massot talking about it last November; since then Riou has finished his refactor of homological algebra so I think we're ready. Both Massot and Riou are at Saclay.
Johan Commelin (Jan 25 2024 at 14:59):
Patrick Massot is Pittsburgh for the rest of this academic year.
Adam Topaz (Jan 25 2024 at 15:00):
There are also lots of people thinking about formalizing infinity category theory, so I’m sure some projects in this field would be both interesting and useful
Patrick Massot (Jan 25 2024 at 15:12):
Bonjour Benoît ! How much time do you want to spend on this? One project that some students here in CMU worked on but did not finish is formalizing Milnor's proof of the hairy ball theorem. It is a geometric proof of an algebraic topology result so it fits your list, and it is much more elementary than infinity category theory. I think it would be a very nice project.
Anatole Dedecker (Jan 25 2024 at 15:52):
Another thing that would be nice would be to help develop the theory of covering maps (if my calculations are correct and if you indeed follow his course, I think Frédéric Paulin should start telling you about it either this week or next week :wink:). But people have been thinking about this so there's a higher collision risk I would say.
Anatole Dedecker (Jan 25 2024 at 15:59):
For example it could be relatively easy and very helpful to build the theory of proper group actions on top of docs#IsProperMap, which will also be somewhat related to Frédéric Paulin's course. That's probably less fun than the hairy ball theorem though!
Adam Topaz (Jan 25 2024 at 16:10):
I'm not familiar with Milnor's proof of the hairy ball theorem, but certainly the proof via the Euler characteristic would introduce various things which are worthwhile to have independently of that theorem.
namibj (Jan 25 2024 at 16:41):
I'm not sure if this is out-of-scope, but formalization should help with verifying the impact of architectural modifications:
https://www.semanticscholar.org/paper/Signal-Propagation-in-Transformers%3A-Theoretical-and-Noci-Anagnostidis/5eeb80dc67590422db64ca95ec0aded24799cfb6
namibj (Jan 25 2024 at 16:43):
(I'd love a classification of this along this sort of schema, though, if anyone would like to teach me.)
Benoît Guillemet (Jan 25 2024 at 16:51):
Thank you for all your answers!
I think the most doable project for us among the ones you proposed is either one of the proofs of the hairy ball theorem or some results in the theory of covering maps. The idea is only to spend a few hours a week in our spare time to have fun with Lean, so even the basics of singular homology seem a little too big. How can I know if people are already working on covering maps?
I will discuss that with the people who want to get into this project with me and keep you informed of what we choose!
Anatole Dedecker (Jan 25 2024 at 17:00):
If I remember correctly, @Junyan Xu was working on this actively (e.g in #7596, which I should go back to reviewing now that my semester is finished). I'll try to find the last thread about it.
Anatole Dedecker (Jan 25 2024 at 17:06):
Here is the thread: https://leanprover.zulipchat.com/#narrow/stream/116395-maths/topic/Path.20lifting
Reading it again it seems that a few people have proven the path/homotopy lifting property already, so it's not a good idea to do one more proof. On the other hand, if we can manage to get that merged relatively soon then you could build on top of it.
Anatole Dedecker (Jan 25 2024 at 17:11):
I think with enough organization we should be able to split the work so that no one steps on other's people toes, if you are interested we could open another thread about it.
Anatole Dedecker (Jan 25 2024 at 17:16):
By the way I'd be really happy to talk about this IRL if you want, whatever you end up working on! Most of my courses are in Paris this semester, but I should still be in Orsay relatively frequently (I'm in M2 AAG).
Scott Carnahan (Jan 26 2024 at 06:23):
Here's an unformalized fact that might go in interesting directions: a "Hopf algebra object" in the category of sets is the same thing as a group. Here, the "comultiplication" is necessarily the diagonal embedding.
Benoît Guillemet (Jan 26 2024 at 16:49):
Anatole Dedecker said:
By the way I'd be really happy to talk about this IRL if you want, whatever you end up working on! Most of my courses are in Paris this semester, but I should still be in Orsay relatively frequently (I'm in M2 AAG).
Thank you for the details. It would indeed be really nice if we could meet you and ask you a few questions IRL (maybe we can talk about this in dm)!
Scott Carnahan said:
Here's an unformalized fact that might go in interesting directions: a "Hopf algebra object" in the category of sets is the same thing as a group. Here, the "comultiplication" is necessarily the diagonal embedding.
Thank you for your proposition!
We finally chose to start with a proof of the hairy ball theorem, but this is only the beginning.
Patrick Massot (Jan 26 2024 at 16:59):
I guess you found it already but the proof I had in mind is https://www.jstor.org/stable/2320860
Junyan Xu (Jan 28 2024 at 08:14):
If you'd like projects around covering spaces and fundamental groups, take a look at the "Planned" tab of the Covering spaces and étale spaces project; I just added a detailed outline towards the Van Kampen theorem. Constructing the monodromy of a covering map and proving the lifting criterion should also be quite straightforward given what's already in #10084. I'm not sure I'll find time to work on them in the near future, but I'll certainly be happy to answer questions and review PRs.
(Update: I've added links to some PRs/branches that I've started but not finished.)
Benoît Guillemet (Jan 28 2024 at 23:27):
Patrick Massot said:
I guess you found it already but the proof I had in mind is https://www.jstor.org/stable/2320860
Thank you! We are currently studying the different proofs to determine which is most interesting for us to formalize.
Junyan Xu said:
If you'd like projects around covering spaces and fundamental groups, take a look at the "Planned" tab of the Covering spaces and étale spaces project; I just added a detailed outline towards the Van Kampen theorem. Constructing the monodromy of a covering map and proving the lifting criterion should also be quite straightforward given what's already in #10084. I'm not sure I'll find time to work on them in the near future, but I'll certainly be happy to answer questions and review PRs.
(Update: I've added links to some PRs/branches that I've started but not finished.)
Thank you for your answer. For the moment, we're going to work on the hairy ball theorem, but we may come back to you later.
Patrick Massot (Jan 29 2024 at 16:34):
Milnor's proof is a cute elementary proof but the downside is that it leaves you with no understanding of why the theorem is true and no tool to prove more results. The principled way of proving this result is to build an algebro-topological invariant that can be computed using any vector field. Say you manage to define the Euler characteristic of a manifold and prove that every vector field which vanishes transversely can be used to compute the Euler characteristic. Then you can compute the Euler characteristic of even-dimensional spheres using your favorite explicit vector field and get and argue that a nowhere vanishing vector field would allow to prove in . But this is a lot more work to formalize than Milnor's proof.
Benoît Guillemet (Jan 30 2024 at 18:51):
Ok, so I guess Milnor's proof should be more reasonable to begin with.
I also found another proof using homology that seems a bit more elementary than the one you described. Assuming there exists a non-vanishing vector field , you could get a homotopy between the identical map and the antipodal map on with . As the degree of the antipodal map is as long as is even, you can derive a contradiction. However, I don't know if the degree of a map is already formalized in Lean or not. It could be quite hard to do depending on what is already in mathlib and what isn't.
Patrick Massot (Jan 30 2024 at 23:34):
This is also a nice proof but indeed it requires degree theory which is not trivial to setup either.
Kevin Cheung (Jan 31 2024 at 12:42):
I would like to see a formalized proof of the Perfect Graph Theorem.
Mauricio Collares (Jan 31 2024 at 14:15):
The Lovász one or the strong one?
Kevin Cheung (Jan 31 2024 at 14:19):
The Strong Perfect Graph Theorem.
Kevin Cheung (Jan 31 2024 at 14:22):
That will probably take years of work though. Maybe the Weak Perfect Graph Theorem is a good start since it's already done in Coq. https://arxiv.org/abs/1912.02211
Benoît Guillemet (Feb 05 2024 at 23:39):
We finally chose to work on Milnor's proof to begin with something simple. We are supervised by @Anatole Dedecker, so everything should go well!
Kevin Cheung said:
I would like to see a formalized proof of the Perfect Graph Theorem.
Thank you for your suggestion. It may be for another project.
Last updated: May 02 2025 at 03:31 UTC