Skip to content

Commit

Permalink
fix simpComm linter
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Nov 18, 2024
1 parent 537fdfa commit 899ed8a
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Batteries/Tactic/Lint/Simp.lean
Original file line number Diff line number Diff line change
Expand Up @@ -228,7 +228,7 @@ private def Expr.eqOrIff? : Expr → Option (Expr × Expr)
noErrorsFound := "No commutativity lemma is marked simp."
errorsFound := "COMMUTATIVITY LEMMA IS SIMP.
Some commutativity lemmas are simp lemmas:"
test := fun declName => withReducible do
test := fun declName => withSimpGlobalConfig do withReducible do
unless ← isSimpTheorem declName do return none
let ty := (← getConstInfo declName).type
forallTelescopeReducing ty fun _ ty' => do
Expand Down

0 comments on commit 899ed8a

Please sign in to comment.