Zulip Chat Archive

Stream: maths

Topic: homotopy theory


Dean Young (Feb 05 2023 at 18:23):

Does mathlib4 have a model category type? I am trying to show that something is Quillen equivalent to CW-complexes.

Yury G. Kudryashov (Feb 05 2023 at 18:25):

Please create a new topic instead of posting to an unrelevant one.

Dean Young (Feb 05 2023 at 18:31):

Does math lib have the homotopy category?

Dean Young (Feb 05 2023 at 18:37):

Can somebody help me out a bit? I am looking for the math lib constructions of

  • homotopy colimits
  • homotopy pullback
  • pi0
  • CW-complexes

Notification Bot (Feb 05 2023 at 18:41):

4 messages were moved here from #mathlib4 > lean4#2074 (new-style structures) by Yury G. Kudryashov.

Yury G. Kudryashov (Feb 05 2023 at 18:42):

@Kind Bubble I moved your messages to a new topic. Please don't post to a random topic next time.

Yury G. Kudryashov (Feb 05 2023 at 18:43):

Did you search for the word "homotopy" in the mathlib repo?

Yury G. Kudryashov (Feb 05 2023 at 18:45):

Note that you should use the Lean 3 version because many "advanced" files were not ported to mathlib 4 yet.

Adam Topaz (Feb 05 2023 at 19:37):

We don't have model categories. But we do have many people who thought about formalizing model categories.

Dean Young (Feb 05 2023 at 19:41):

What about a model of the homotopy category?

Adam Topaz (Feb 05 2023 at 19:42):

What do you want exactly?

Dean Young (Feb 05 2023 at 19:42):

Preferably CW-complexes.

Adam Topaz (Feb 05 2023 at 19:43):

We don't have CW complexes

Dean Young (Feb 05 2023 at 19:44):

What about point-set topological spaces?

Adam Topaz (Feb 05 2023 at 19:44):

Yes, we have those of course. We also have geometric realizations of simplicial sets.

Dean Young (Feb 05 2023 at 19:45):

can you give me a link to where this is built up? Is there a point-set-topological-space-for-Lean tutorial?

Adam Topaz (Feb 05 2023 at 19:45):

If you can explain what you're trying to prove more precisely, then it would be easier to say whether it is feasible or not

Adam Topaz (Feb 05 2023 at 19:45):

docs#topological_space

Adam Topaz (Feb 05 2023 at 19:45):

Your lean experience would be much smoother if you figure out how to use the api search

Adam Topaz (Feb 05 2023 at 19:46):

https://leanprover-community.github.io/mathlib_docs

Dean Young (Feb 05 2023 at 19:47):

Thanks so much Adam. What's the API search?

Adam Topaz (Feb 05 2023 at 19:48):

See the last link above

Dean Young (Feb 05 2023 at 19:49):

I have a model for the homotopy category- that much is already done. But the main goal is to show quillen equivalence with whatever the most mainstream one is.

Adam Topaz (Feb 05 2023 at 19:50):

I think the category of simplicial sets would be the most natural choice for that

Adam Topaz (Feb 05 2023 at 19:50):

docs#sSet

Adam Topaz (Feb 05 2023 at 19:51):

What model did you construct?

Dean Young (Feb 05 2023 at 20:32):

I think with simplicial sets I would need recourse to topological spaces unless I restricted to the ones which have the lifting conditions of an ∞-groupoid. Whitehead's theorem and the cellular approximation theorem are major milestones. Unfortunately the model I made is kind of involved so I can't describe it at the moment. Usually they involve something which demands that the space of double base point preserving maps f: [0, 1] -> [0, 1] v ... v [0, 1] is contractible.

Adam Topaz (Feb 05 2023 at 20:33):

Stating the infinity groupoid condition is easy, since we have horns already in mathlib. As I said above, we also have the geometric realization functor from sSet to Top

Adam Topaz (Feb 05 2023 at 20:34):

The whole formalism necessary to state the concept of a Quillen adjunction still needs to be developed though.

Reid Barton (Feb 05 2023 at 22:19):

See also https://github.com/rwbarton/lean-model-categories/tree/top-dev which got most of the way through constructing the model category Top, but it's for an ancient version of mathlib

Joël Riou (Feb 12 2023 at 22:27):

In https://github.com/joelriou/homotopical_algebra/tree/main/src/for_mathlib/algebraic_topology/homotopical_algebra, I have obtained some basic results on model categories, like the fundamental lemma of homotopical algebra (computation of morphisms in the localized category using homotopy classes of morphisms...). I have been thinking recently about total (left/right) derived functors, so that stating what a Quillen adjunction is should not be very hard. However, proving that there is a Quillen equivalence requires that we already know both categories are model categories... I am afraid the hardest parts should be more about constructing these model category structures rather than about getting an equivalence. I would suggest starting with topological spaces (or compactly generated hausdorff spaces?).


Last updated: Dec 20 2023 at 11:08 UTC