Zulip Chat Archive
Stream: mathlib4
Topic: terminal.comp_from_assoc
Charlie Conneen (Feb 07 2025 at 00:28):
In CategoryTheory.Limits.Shapes.Terminal:
@[simp]
theorem terminal.comp_from [HasTerminal C] {P Q : C} (f : P ⟶ Q) :
f ≫ terminal.from Q = terminal.from P := by
simp [eq_iff_true_of_subsingleton]
Should this be tagged as reassoc? (Similarly for initial.to_comp)
Charlie Conneen (Feb 07 2025 at 00:31):
Admittedly it's probably not often that one is mapping out of the terminal object, but this has proven to be a significant use case.
Notification Bot (Feb 07 2025 at 00:44):
This topic was moved here from #mathlib4 > terminal.comp_from by Charlie Conneen.
Andrew Yang (Feb 07 2025 at 01:39):
Most probably yes.
Charlie Conneen (Feb 07 2025 at 02:23):
It seems that initial.to_comp_assoc does not need to be a simp lemma. I have opted to simply not add the reassoc tag to initial.to_comp. PR is here: #21527
Andrew Yang (Feb 07 2025 at 03:06):
An assoc version of initial.to_comp might still be useful though. Perhaps add the assocbut without taging the assoc as simp? (You can achieve this by @[simp, reassoc] instead of @[reassoc (attr := simp)])
Charlie Conneen (Feb 07 2025 at 03:07):
Ah, sure. Thanks for input.
Last updated: May 02 2025 at 03:31 UTC