batteries icon indicating copy to clipboard operation
batteries copied to clipboard

`simpNF` should use dsimp for lemmas proved by `rfl`

Open digama0 opened this issue 2 years ago • 1 comments

The @[simp] attribute is used by both simp and dsimp, so it is possible for a rfl lemma to have a proof by simp but not one by dsimp, and so this is a false positive. The linter should check if the current declaration is a rfl lemma and if so restrict its attention to dsimp proofs.

digama0 avatar Jan 13 '23 08:01 digama0

I've just updated the links in mathlib4 pointing to mathlib4#5081 to point to this issue instead.

This link searches for references to this issue in the mathlib4 source code.

kim-em avatar Aug 06 '23 00:08 kim-em