Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.expandNextGoal.fmt
{Q : Type}
[Aesop.Queue Q]
(id : Aesop.GoalId)
(priority : Aesop.Percent)
(initialGoal : Lean.MVarId)
(initialMetaState : Lean.Meta.SavedState)
(result : Except Lean.Exception Aesop.RuleResult)
 :
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.expandNextGoal.traceNewRapps
{Q : Type}
[Aesop.Queue Q]
(newRapps : Array Aesop.RappRef)
 :
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
Equations
- Aesop.getProof? = do let __do_lift ← liftM Aesop.getRootMVarId Lean.getExprMVarAssignment? __do_lift
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.checkRenderedScript
{Q : Type}
[Aesop.Queue Q]
(completeProof : Bool)
(script : Lean.TSyntax `Lean.Parser.Tactic.tacticSeq)
 :
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.structureScript
{Q : Type}
[Aesop.Queue Q]
(uscript : Aesop.Script.UScript)
(rootState : Lean.Meta.SavedState)
(rootGoal : Lean.MVarId)
 :
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
- Aesop.traceTree = do let __do_lift ← liftM Aesop.getRootGoal let __do_lift ← ST.Ref.get __do_lift liftM (__do_lift.traceTree Aesop.TraceOption.tree)
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
This function detects whether the search has made progress, meaning that the remaining goals after safe prefix expansion are different from the initial goal. We approximate this by checking whether, after safe prefix expansion, either of the following statements is true.
- There is a safe rapp.
- A subgoal of the preprocessing rule has been modified during normalisation.
This is an approximation because a safe rule could, in principle, leave the initial goal unchanged.
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.throwAesopEx
{Q : Type}
[Aesop.Queue Q]
{α : Type}
(mvarId : Lean.MVarId)
(remainingSafeGoals : Array Lean.MVarId)
(safePrefixExpansionSuccess : Bool)
(msg? : Option Lean.MessageData)
 :
Aesop.SearchM Q α
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.search
(goal : Lean.MVarId)
(ruleSet? : optParam (Option Aesop.LocalRuleSet) none)
(options : optParam Aesop.Options
  { strategy := Aesop.Strategy.bestFirst, maxRuleApplicationDepth := 30, maxRuleApplications := 200, maxGoals := 0,
    maxNormIterations := 100, maxSafePrefixRuleApplications := 50, maxRuleHeartbeats := 0, maxSimpHeartbeats := 0,
    maxUnfoldHeartbeats := 0, applyHypsTransparency := Lean.Meta.TransparencyMode.default,
    assumptionTransparency := Lean.Meta.TransparencyMode.default,
    destructProductsTransparency := Lean.Meta.TransparencyMode.reducible, introsTransparency? := none,
    terminal := false, warnOnNonterminal := true, traceScript := false, enableSimp := true, useSimpAll := true,
    useDefaultSimpSet := true, enableUnfold := true })
(simpConfig : optParam Lean.Meta.Simp.Config
  { maxSteps := Lean.Meta.Simp.defaultMaxSteps, maxDischargeDepth := 2, contextual := false, memoize := true,
    singlePass := false, zeta := true, beta := true, eta := true, etaStruct := Lean.Meta.EtaStructMode.all,
    iota := true, proj := true, decide := false, arith := false, autoUnfold := false, dsimp := true,
    failIfUnchanged := true, ground := false, unfoldPartialApp := false, zetaDelta := false, index := true })
(simpConfigSyntax? : optParam (Option Lean.Term) none)
(stats : optParam Aesop.Stats ∅)
 :
Equations
- One or more equations did not get rendered due to their size.