Zulip Chat Archive

Stream: general

Topic: Is this a good simp lemma?


Gabriel Ebner (Feb 24 2020 at 11:04):

We have a lot of simp lemmas of the following form:

@[simp] lemma foo : bar = baz := by simp

Is this ever useful? Were these intentional?

Mario Carneiro (Feb 24 2020 at 11:43):

they are shortcut rules

Mario Carneiro (Feb 24 2020 at 11:44):

I know why you are asking, but since it's confluent it doesn't matter if the lemma triggers or not

Mario Carneiro (Feb 24 2020 at 11:45):

maybe just nolint them

Gabriel Ebner (Feb 24 2020 at 12:40):

they are shortcut rules

So I guess I'll just rewrite the linter and check that (i.e. that they are indeed used preferentially). Putting nolint is not really an option since they are lots of these lemmas.


Last updated: Dec 20 2023 at 11:08 UTC