Zulip Chat Archive

Stream: mathlib4

Topic: !4#3705 (Topology.Category.Profinite.Basic)


Scott Morrison (Apr 28 2023 at 12:03):

!4#3705 (Topology.Category.Profinite.Basic) is hopefully not far from done. Some simp lemmas must be missing at the remaining sorries, because the goal is not as nice as the corresponding point in mathlib3.

If any of the "Profinite people" (@Kevin Buzzard, @Adam Topaz?) would like to take over this one I'm done for the day.

Adam Topaz (Apr 28 2023 at 12:52):

I don’t think I’m totally disconnected, but I can take a look in a couple of hours anyway ;)

Adam Topaz (Apr 28 2023 at 14:05):

Okay, I got the file to build by adding the following lemma:

-- Porting note: This lemma was not needed in mathlib3
@[simp]
lemma forget_ContinuousMap_mk {X Y : Profinite} (f : X  Y) (hf : Continuous f) :
    (forget Profinite).map (ContinuousMap.mk f hf) = f :=
  rfl

Presumably the changes to start-port.sh should be split off to a separate PR?

Adam Topaz (Apr 28 2023 at 14:06):

I think a similar lemma would be helpful for TopCat and CompHaus as well.

Matthew Ballard (Apr 28 2023 at 14:11):

Yeah that is a good idea

Adam Topaz (Apr 28 2023 at 14:12):

In the long run (i.e. after the port) I think we should make homs in concrete categories such as Type, TopCat, etc. into structures so lean doesn't get so easily confused about when something should be a morphism and when it should be a function/continuousMap

Adam Topaz (Apr 28 2023 at 15:00):

Well, it looks like we still have some linting errors. I think the simp lemmas around coercions to functions need to be shuffled a bit.


Last updated: Dec 20 2023 at 11:08 UTC