Skip to content

Commit

Permalink
chore: simproc PR changes (#496)
Browse files Browse the repository at this point in the history
See leanprover/lean4#3124

Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
  • Loading branch information
2 people authored and joehendrix committed Feb 5, 2024
1 parent 19abd0c commit 89fe00d
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Std/Lean/Meta/Simp.lean
Original file line number Diff line number Diff line change
Expand Up @@ -58,7 +58,7 @@ def mkSimpContext' (simpTheorems : SimpTheorems) (stx : Syntax) (eraseLocal : Bo
let r ← elabSimpArgs stx[4] (eraseLocal := eraseLocal) (kind := kind) (simprocs := #[simprocs]) {
config := (← elabSimpConfig stx[1] (kind := kind))
simpTheorems := #[simpTheorems], congrTheorems
}
} simprocs
if !r.starArg || ignoreStarArg then
return { r with dischargeWrapper }
else
Expand Down

0 comments on commit 89fe00d

Please sign in to comment.