Zulip Chat Archive
Stream: mathlib4
Topic: where to place bicategory lemma
Calle Sönne (Jun 09 2024 at 17:55):
I need the following lemma (about Oplax functors) in an upcoming PR:
lemma map₂_eqToHom {a b : B} {f g : a ⟶ b} (h : f = g) :
F.map₂ (eqToHom h) = eqToHom (F.congr_map h) := by
subst h; simp only [eqToHom_refl, OplaxFunctor.map₂_id]
I'm not sure where to place it, as Bicategory/Functor
currently does not import eqToHom
and I'm worried this will add a lot of imports that are not really needed there. It also feels weird to add a new file Bicategory/eqToHom
just for this one lemma. Does anyone have any recommendations?
Kevin Buzzard (Jun 09 2024 at 18:54):
I think the community is moving on from the weird feelings and is now rather disposed to having lots of small files.
Adam Topaz (Jun 09 2024 at 20:40):
I think a natural place might be the file about locally discrete bicats
Calle Sönne (Jun 10 2024 at 09:35):
Adam Topaz said:
I think a natural place might be the file about locally discrete bicats
Okay that sound reasonable
Last updated: May 02 2025 at 03:31 UTC