Zulip Chat Archive
Stream: mathlib4
Topic: Broken line breaking in mathport output
Ruben Van de Velde (May 31 2023 at 08:58):
https://github.com/leanprover-community/mathlib3port/commit/6797a637bad89c884a1ea52371e5256b851945f5 improved output in a lot of places, but it also started using syntax like
@[ext]
theorem cokernel_π_imageSubobject_ext {L M N : ModuleCat.{v} R} (f : L ⟶ M) [HasImage f]
(g : (imageSubobject f : ModuleCat.{v} R) ⟶ N) [HasCokernel g] {x y : N} (l : L)
(w : x = y + g (factorThruImageSubobject f l)) : cokernel.π g x = cokernel.π g y := by subst w;
simp
which doesn't work. Not sure what caused this or who should look at it
Last updated: Dec 20 2023 at 11:08 UTC