Skip to content

Commit 5920aea

Browse files
Merge main into nightly-testing
2 parents ca6423f + 6ac5303 commit 5920aea

File tree

1 file changed

+4
-2
lines changed

1 file changed

+4
-2
lines changed

Batteries/Tactic/Lint/Simp.lean

Lines changed: 4 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -102,8 +102,10 @@ def formatLemmas (usedSimps : Simp.UsedSimps) (simpName : String) (higherOrder :
102102
@[env_linter] def simpNF : Linter where
103103
noErrorsFound := "All left-hand sides of simp lemmas are in simp-normal form."
104104
errorsFound := "SOME SIMP LEMMAS ARE NOT IN SIMP-NORMAL FORM.
105-
see note [simp-normal form] for tips how to debug this.
106-
https://leanprover-community.github.io/mathlib_docs/notes.html#simp-normal%20form"
105+
Please change the lemma to make sure their left-hand sides are in simp normal form.
106+
To learn about simp normal forms, see
107+
https://leanprover-community.github.io/extras/simp.html#simp-normal-form
108+
and https://lean-lang.org/doc/reference/latest/The-Simplifier/Simp-Normal-Forms/."
107109
test := fun declName => do
108110
unless ← isSimpTheorem declName do return none
109111
withConfig Elab.Term.setElabConfig do

0 commit comments

Comments
 (0)