- options : Options'
- ruleSet : LocalRuleSet
- normSimpContext : NormSimpContext
- statsRef : StatsRef
Instances For
@[reducible, inline]
Equations
Instances For
Equations
- Aesop.instMonadBacktrackSavedStateNormM = { saveState := liftM Lean.Meta.saveState, restoreState := fun (s : Lean.Meta.SavedState) => liftM s.restore }
Equations
- Aesop.instMonadStatsNormM = Aesop.MonadStats.mk do let __do_lift ← read pure __do_lift.statsRef
- succeeded (goal : Lean.MVarId) (steps? : Option (Array Script.LazyStep)) : NormRuleResult
- proved (steps? : Option (Array Script.LazyStep)) : NormRuleResult
Instances For
Equations
- (Aesop.NormRuleResult.succeeded goal steps?).newGoal? = some goal
- (Aesop.NormRuleResult.proved steps?).newGoal? = none
Instances For
Equations
- (Aesop.NormRuleResult.succeeded goal steps?).steps? = steps?
- (Aesop.NormRuleResult.proved steps?).steps? = steps?
Instances For
Equations
Instances For
@[always_inline]
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.withNormTraceNode.fmt
(ruleName : DisplayRuleName)
(r : Except Lean.Exception (Option NormRuleResult))
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.runNormRuleTac.err
(rule : NormRule)
(input : RuleTacInput)
{α : Type}
(msg : Lean.MessageData)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.runNormRule
(goal : Lean.MVarId)
(mvars : UnorderedArraySet Lean.MVarId)
(rule : IndexMatchResult NormRule)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.runFirstNormRule
(goal : Lean.MVarId)
(mvars : UnorderedArraySet Lean.MVarId)
(rules : Array (IndexMatchResult NormRule))
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.mkNormSimpScriptStep
(preGoal : Lean.MVarId)
(postGoal? : Option Lean.MVarId)
(preState postState : Lean.Meta.SavedState)
(usedTheorems : Lean.Meta.Simp.UsedSimps)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.SimpResult.toNormRuleResult
(originalGoal : Lean.MVarId)
(preState postState : Lean.Meta.SavedState)
:
Equations
- One or more equations did not get rendered due to their size.
- Aesop.SimpResult.toNormRuleResult originalGoal preState postState Aesop.SimpResult.unchanged = pure none
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.normSimpCore.addLocalRules
(goal : Lean.MVarId)
(localRules : Array LocalNormSimpRule)
(ctx : Lean.Meta.Simp.Context)
(simprocs : Lean.Meta.Simp.SimprocsArray)
(isSimpAll : Bool)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[always_inline]
def
Aesop.checkSimp
(name : String)
(mayCloseGoal : Bool)
(goal : Lean.MVarId)
(x : NormM (Option NormRuleResult))
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
- proved (script : Array (DisplayRuleName × Option (Array Script.LazyStep))) : NormSeqResult
- changed (goal : Lean.MVarId) (script : Array (DisplayRuleName × Option (Array Script.LazyStep))) : NormSeqResult
- unchanged : NormSeqResult
Instances For
Equations
- Aesop.NormRuleResult.toNormSeqResult ruleName (Aesop.NormRuleResult.proved steps?) = Aesop.NormSeqResult.proved #[(ruleName, steps?)]
- Aesop.NormRuleResult.toNormSeqResult ruleName (Aesop.NormRuleResult.succeeded goal steps?) = Aesop.NormSeqResult.changed goal #[(ruleName, steps?)]
Instances For
@[reducible, inline]
Equations
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Aesop.NormStep.runPreSimpRules mvars x✝² x✝¹ x✝ = Aesop.optNormRuleResultToNormSeqResult <$> Aesop.runFirstNormRule x✝² mvars x✝¹
Instances For
Equations
- Aesop.NormStep.runPostSimpRules mvars x✝² x✝¹ x✝ = Aesop.optNormRuleResultToNormSeqResult <$> Aesop.runFirstNormRule x✝² mvars x✝
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.