Skip to content

Commit

Permalink
fix: unset trailing for simpa? "try this" suggestion (#5907)
Browse files Browse the repository at this point in the history
Closes #4581
  • Loading branch information
kmill authored Nov 8, 2024
1 parent 9b167e2 commit 85f2213
Showing 1 changed file with 2 additions and 1 deletion.
3 changes: 2 additions & 1 deletion src/Lean/Elab/Tactic/Simpa.lean
Original file line number Diff line number Diff line change
Expand Up @@ -95,7 +95,8 @@ deriving instance Repr for UseImplicitLambdaResult
else
g.assumption; pure stats
if tactic.simp.trace.get (← getOptions) || squeeze.isSome then
let stx ← match ← mkSimpOnly stx stats.usedTheorems with
let usingArg : Option Term := usingArg.map (⟨·.raw.unsetTrailing⟩)
let stx ← match ← mkSimpOnly stx.raw.unsetTrailing stats.usedTheorems with
| `(tactic| simp $cfg:optConfig $(disch)? $[only%$only]? $[[$args,*]]?) =>
if unfold.isSome then
`(tactic| simpa! $cfg:optConfig $(disch)? $[only%$only]? $[[$args,*]]? $[using $usingArg]?)
Expand Down

0 comments on commit 85f2213

Please sign in to comment.