Skip to content

Commit

Permalink
chore: adapt to decide := false in simp
Browse files Browse the repository at this point in the history
  • Loading branch information
collares committed Oct 23, 2023
1 parent 9dc4a10 commit e6d2c12
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 2 deletions.
2 changes: 1 addition & 1 deletion Aesop/Options/Public.lean
Original file line number Diff line number Diff line change
Expand Up @@ -115,7 +115,7 @@ structure Options where
/--
Options which modify the behaviour of the builtin `simp` normalisation rule.
Extends `Lean.Meta.Simp.ConfigCtx`, so any option declared there is also valid
here. For example, you can use `aesop (simp_config := { arith := true })` to get
here. For example, you can use `aesop (simp_options := { arith := true })` to get
behaviour similar to `simp (config := { arith := true })` (aka `simp_arith`).
-/
structure SimpConfig extends Lean.Meta.Simp.ConfigCtx where
Expand Down
2 changes: 1 addition & 1 deletion Aesop/Search/Expansion/Norm.lean
Original file line number Diff line number Diff line change
Expand Up @@ -377,7 +377,7 @@ partial def normalizeGoalMVar (rs : RuleSet) (normSimpContext : NormSimpContext)
NormStep.simp rs normSimpContext options mvarsHashSet,
NormStep.runPostSimpRules options mvars
]
runNormSteps rs goal options.maxNormIterations normSteps (by simp)
runNormSteps rs goal options.maxNormIterations normSteps (by simp (config := { decide := true }))

-- Returns true if the goal was solved by normalisation.
def normalizeGoalIfNecessary (gref : GoalRef) [Aesop.Queue Q] :
Expand Down

0 comments on commit e6d2c12

Please sign in to comment.