Zulip Chat Archive

Stream: general

Topic: slow elaboration with bundled homomorphisms


Yury G. Kudryashov (Jul 12 2020 at 04:46):

here adding by simpa only [] makes elaboration much faster. I have no idea why. Here is the code:

lemma function.injective.has_sum_iff {g : γ  β} (hg : injective g)
  (hf :  x  set.range g, f x = 0) :
  has_sum (f  g) a  has_sum f a :=
by simpa only [] using function.embedding.has_sum_iff g, hg hf

This is a part of #3371.

Yury G. Kudryashov (Jul 12 2020 at 04:47):

another example

Sebastien Gouezel (Jul 12 2020 at 08:15):

Did you know that you can remove the [] in by simpa only []?


Last updated: Dec 20 2023 at 11:08 UTC