Zulip Chat Archive
Stream: Copenhagen Masterclass 2023
Topic: TFAE fam of epis
Boris Kjær (Jun 26 2023 at 11:14):
Here's to work on TFAE statement regarding finite families of epimorphisms in ProFinite and ExtrDisc
Boris Kjær (Jun 26 2023 at 11:28):
Created branch bbolvig/families-of-effective-epis
Riccardo Brasca (Jun 26 2023 at 11:32):
Can you push a sorried statement? We need it to prove that Profinite
is precoherent
Riccardo Brasca (Jun 26 2023 at 11:33):
Well, in practice we are doing the same thing... are you working on it?
Boris Kjær (Jun 26 2023 at 11:36):
yes, the statement has been added in Profinite/Epi.lean
Boris Kjær (Jun 26 2023 at 11:47):
Is that working for you guys?
Riccardo Brasca (Jun 26 2023 at 11:48):
Yes thanks
Riccardo Brasca (Jun 26 2023 at 11:49):
For profinite
variable {X Y B : Profinite.{u}} (f : X ⟶ B) (g : Y ⟶ B)
/--
The pullback of two morphisms `f,g` in `Profinite`, constructed explicitly as the set of
pairs `(x,y)` such that `f x = g y`, with the topology induced by the product.
-/
def pullback : Profinite.{u} :=
letI set := { xy : X × Y | f xy.fst = g xy.snd }
haveI : CompactSpace set := by
rw [← isCompact_iff_compactSpace]
apply IsClosed.isCompact
exact isClosed_eq (f.continuous.comp continuous_fst) (g.continuous.comp continuous_snd)
Profinite.of set
works
Riccardo Brasca (Jun 26 2023 at 11:49):
I think you also need it
Jon Eugster (Jun 26 2023 at 18:29):
totally golfed code ;)
intro x hx y hy
unfold Set.Subsingleton at h
have a₁ : (f.inv x) ∈ ↑f.hom ⁻¹' t
· rw [Set.mem_preimage]
simpa
have a₂ : (f.inv y) ∈ ↑f.hom ⁻¹' t
· rw [Set.mem_preimage]
simpa
specialize h a₁ a₂
replace h := congr_arg f.hom h
simp at h
assumption
Jon Eugster (Jun 27 2023 at 10:47):
Template with the statements:
https://github.com/adamtopaz/CopenhagenMasterclass2023/pull/9
@Riccardo Brasca
Riccardo Brasca (Jun 27 2023 at 10:47):
Thanks!
Last updated: Dec 20 2023 at 11:08 UTC