Skip to content

Commit 69497e4

Browse files
committed
m!
1 parent 47423df commit 69497e4

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

src/Lean/Meta/Tactic/Simp/Rewrite.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -227,7 +227,7 @@ where
227227
let isRflOld ← withOptions (experimental.tactic.simp.useRflAttr.set · false) do
228228
isRflProof thm.proof
229229
if isRflOld then
230-
logWarning "theorem {thm.proof} is no longer rfl"
230+
logWarning m!"theorem {thm.proof} is no longer rfl"
231231
continue
232232
if let some result ← tryTheoremWithExtraArgs? e thm numExtraArgs then
233233
trace[Debug.Meta.Tactic.simp] "rewrite result {e} => {result.expr}"

0 commit comments

Comments
 (0)