Zulip Chat Archive
Stream: new members
Topic: Confused by "simp_nf linter" error
Sebastian Monnet (Apr 27 2022 at 15:50):
My PR #13307 is failing the "Lint mathlib" check, because apparently the lemma inclusion_right
in algebra/algebra/subalgebra/basic
can be proved by simp. I can see why this is undesirable, since the lemma is a simp lemma, so this makes it kind of redundant. I have two problems, however:
1) As far as I can tell, my PR doesn't change any files that subalgebra/basic
depends on, so I don't understand why the changes of the PR are triggering the error
2) I'm not sure what the appropriate response is - should I just delete the lemma that's causing the problem?
Yaël Dillies (Apr 27 2022 at 15:57):
This is just because I added the more powerful simp lemma inclusion_mk
, which proves inclusion_right
. I'm getting a PR out to add those lemmas everywhere and unsimp the now redundant lemmas. Hold tight.
Sebastian Monnet (Apr 27 2022 at 16:03):
Yaël Dillies said:
This is just because I added the more powerful simp lemma
inclusion_mk
, which provesinclusion_right
. I'm getting a PR out to add those lemmas everywhere and unsimp the now redundant lemmas. Hold tight.
Okay, thanks!
Last updated: Dec 20 2023 at 11:08 UTC