Zulip Chat Archive

Stream: Copenhagen Masterclass 2023

Topic: Mathlib4 PRs


Adam Topaz (May 30 2023 at 16:34):

!4#4505

Adam Topaz (May 30 2023 at 16:34):

@Dagur Ásgeirsson @Kevin Buzzard

Scott Morrison (May 31 2023 at 00:43):

:octopus: and :tada: are nice, I guess, but how about a review? :-)

Filippo A. E. Nuccio (May 31 2023 at 08:08):

I have started one.

Adam Topaz (May 31 2023 at 14:38):

Thanks @Filippo A. E. Nuccio I'll take a look soon.

Anyway, here's a bit of additional motivation ;) !4#4527 (this last PR still needs some work, but the main constructions are there)

Filippo A. E. Nuccio (May 31 2023 at 14:39):

I'll have a look at that one as well.

Adam Topaz (May 31 2023 at 14:39):

Thanks, but I'm still working on this one. I need to move some things to the right place.

Filippo A. E. Nuccio (May 31 2023 at 14:40):

Oh, I see. Then I will wait and then have a look :smile: :hourglass:

Adam Topaz (May 31 2023 at 14:43):

Maybe a quick summary of this last PR: It has two key results:

theorem effectiveEpiFamily_tfae
    {α : Type} [Fintype α] {B : CompHaus.{u}}
    (X : α  CompHaus.{u}) (π : (a : α)  (X a  B)) :
    [ EffectiveEpiFamily X π
    , Epi (Sigma.desc π)
    ,  b : B,  (a : α) (x : X a), π a x = b
    ].TFAE :=

and

instance : Precoherent CompHaus.{u} :=

And, of course, as a result:

namespace Condensed

def Condensed.{u} (C : Type _) [Category C] :=
  Sheaf (CoherentTopology CompHaus.{u}) C

instance {C : Type _} [Category C] : Category (Condensed.{u} C) :=
  show Category (Sheaf _ _) from inferInstance

end Condensed

Adam Topaz (May 31 2023 at 14:45):

At some point someone should write down a definition of coherent categories, and show that CompHaus is actually coherent (and that coherent implies precoherent)

Adam Topaz (Jun 01 2023 at 17:58):

!4#4527 should be ready for review (@Johan Commelin @Dagur Ásgeirsson @Kevin Buzzard )

Adam Topaz (Jun 01 2023 at 18:00):

I would have pinged you too Filippo, but you had already said you would review it ;)

Adam Topaz (Jun 01 2023 at 18:04):

Oh, I should add some refs in the condensed file... let me do that now.

Adam Topaz (Jun 01 2023 at 18:16):

refs added!

Dagur Asgeirsson (Jun 01 2023 at 23:54):

I’ll take a look in the morning! Don’t know if I’m a qualified reviewer though 😅

Adam Topaz (Jun 09 2023 at 14:40):

Next one is up: !4#4909

Dagur Asgeirsson (Jul 07 2023 at 15:53):

I've opened #5761, #5762, #5763

Dagur Asgeirsson (Jul 07 2023 at 15:54):

Once David's PR is done we can add more to the ExtrDisc folder and start working on getting the explicit descriptions of condensed sets into mathlib

Riccardo Brasca (Jul 07 2023 at 15:57):

Thanks! If you are in the mood of opening PR we have the comparison between product/coproduct in the opposite category that can go to mathlib

Riccardo Brasca (Jul 07 2023 at 15:57):

But I can do it during the weekend

Adam Topaz (Jul 07 2023 at 16:23):

I left a few comments.

Dagur Asgeirsson (Jul 07 2023 at 18:27):

@Riccardo Brasca I’m away over the weekend so you can do it 😅 also feel free to address Adam’s comments. But if you don’t have time I’ll do it on Monday

Dagur Asgeirsson (Jul 09 2023 at 22:56):

Adam Topaz said:

I left a few comments.

Thanks for the suggestions. I've pushed revised versions of all three PR's.

Dagur Asgeirsson (Jul 11 2023 at 10:19):

I added more to the ExtrDisc/Basic file, depending on Gleason: #5808

Dagur Asgeirsson (Jul 13 2023 at 10:11):

@Jon Eugster @Boris Kjær I've opened #5858, planning to do the same for ExtrDisc

Dagur Asgeirsson (Jul 13 2023 at 10:14):

It's Profinite/Epi and Profinite/Coherent from the Copenhagen repo put together into one file Mathlib/Topology/Category/Profinite/EffectiveEpi

Jon Eugster (Jul 13 2023 at 10:17):

Thx! I can fix all the stylistic things on that PR tonight or tomorrow. and also add Sina & Nima as coauthors

Dagur Asgeirsson (Jul 13 2023 at 10:18):

Ok great! I just looked at the commit history when I wrote the list of coauthors

Dagur Asgeirsson (Jul 13 2023 at 10:23):

I've already fixed the style errors the linter gave, if that's what you're talking about

Dagur Asgeirsson (Jul 13 2023 at 11:45):

#5861

Jon Eugster (Jul 13 2023 at 14:12):

I pushed the the cleanups I was thinking about to both PRs. Mostly whitespaces, docstrings and such

Dagur Asgeirsson (Aug 28 2023 at 10:51):

All the sorry-free files in the Copenhagen repo have been PR-ed to mathlib. All the content is in two PR's: #6731 and #6810, which depend on some smaller PR's. Reviews are very welcome! In particular, those that are in need of review right now are: #6750, #6774, #6779 and #6810.

Dagur Asgeirsson (Aug 28 2023 at 10:56):

I should say that the code in #6731 still needs to be cleaned up a lot, but the rest of the file depends on #6750 which I would like others' opinion on before continuing

Riccardo Brasca (Aug 29 2023 at 08:37):

@Dagur Asgeirsson I am still on vacation without a computer, I will have a look on Friday, but thanks a lot for all the work!

Dagur Asgeirsson (Aug 30 2023 at 14:49):

#6876 now makes a lot of the original code triplication redundant. It defines regular and extensive categories, the regular and extensive topologies and proves that their union generates the coherent topology for precoherent, regular and extensive categories.

Dagur Asgeirsson (Oct 09 2023 at 08:27):

#6810, #6877, and #6919 are ready for review, and I think #7421 can be merged

Johan Commelin (Oct 09 2023 at 11:14):

I merged #7421 and left a comment on #6877. Maybe others can chime in on the other 2 PRs?

Johan Commelin (Oct 09 2023 at 11:14):

I need to run to my next meeting.

Dagur Asgeirsson (Nov 20 2023 at 22:23):

The explicit description (#6731) is now finally ready for review!

Johan Commelin (Nov 21 2023 at 04:51):

Left a comment about namespaces


Last updated: Dec 20 2023 at 11:08 UTC