- proved (newRapps : Array RappRef) : RuleResult
- succeeded (newRapps : Array RappRef) : RuleResult
- failed : RuleResult
Instances For
Equations
- (Aesop.RuleResult.proved newRapps).toEmoji = Aesop.ruleProvedEmoji
- (Aesop.RuleResult.succeeded newRapps).toEmoji = Aesop.ruleSuccessEmoji
- Aesop.RuleResult.failed.toEmoji = Aesop.ruleFailureEmoji
Instances For
Equations
- (Aesop.RuleResult.proved newRapps).isSuccessful = true
- (Aesop.RuleResult.succeeded newRapps).isSuccessful = true
- Aesop.RuleResult.failed.isSuccessful = false
Instances For
- regular (result : RuleResult) : SafeRuleResult
- postponed (result : PostponedSafeRule) : SafeRuleResult
Instances For
Equations
- (Aesop.SafeRuleResult.regular r).toEmoji = r.toEmoji
- (Aesop.SafeRuleResult.postponed result).toEmoji = Aesop.rulePostponedEmoji
Instances For
Equations
- (Aesop.SafeRuleResult.regular r).isSuccessfulOrPostponed = r.isSuccessful
- (Aesop.SafeRuleResult.postponed result).isSuccessfulOrPostponed = true
Instances For
def
Aesop.runRegularRuleTac
(goal : Goal)
(tac : RuleTac)
(ruleName : RuleName)
(indexMatchLocations : Std.HashSet IndexMatchLocation)
(patternInstantiations : Std.HashSet RulePatternInstantiation)
(options : Options')
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.addRapps
{Q : Type}
[Queue Q]
(parentRef : GoalRef)
(rule : RegularRule)
(rapps : Array RuleApplication)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[always_inline]
def
Aesop.withRuleTraceNode
{Q : Type}
[Queue Q]
{α : Type}
(ruleName : RuleName)
(toEmoji : α → String)
(suffix : String)
(k : SearchM Q α)
:
SearchM Q α
Equations
- Aesop.withRuleTraceNode ruleName toEmoji suffix k = Aesop.withAesopTraceNode Aesop.TraceOption.steps (Aesop.withRuleTraceNode.fmt ruleName toEmoji suffix) k
Instances For
def
Aesop.withRuleTraceNode.fmt
{Q : Type}
[Queue Q]
{α : Type}
(ruleName : RuleName)
(toEmoji : α → String)
(suffix : String)
(result : Except Lean.Exception α)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.runRegularRuleCore
{Q : Type}
[Queue Q]
(parentRef : GoalRef)
(rule : RegularRule)
(indexMatchLocations : Std.HashSet IndexMatchLocation)
(patternInstantiations : Std.HashSet RulePatternInstantiation)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.runSafeRule
{Q : Type}
[Queue Q]
(parentRef : GoalRef)
(matchResult : IndexMatchResult SafeRule)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.runUnsafeRule
{Q : Type}
[Queue Q]
(parentRef : GoalRef)
(matchResult : IndexMatchResult UnsafeRule)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
- proved (newRapps : Array RappRef) : SafeRulesResult
- succeeded (newRapps : Array RappRef) : SafeRulesResult
- failed (postponed : Array PostponedSafeRule) : SafeRulesResult
- skipped : SafeRulesResult
Instances For
Equations
- (Aesop.SafeRulesResult.proved newRapps).toEmoji = Aesop.ruleProvedEmoji
- (Aesop.SafeRulesResult.succeeded newRapps).toEmoji = Aesop.ruleSuccessEmoji
- (Aesop.SafeRulesResult.failed postponed).toEmoji = Aesop.ruleFailureEmoji
- Aesop.SafeRulesResult.skipped.toEmoji = Aesop.ruleSkippedEmoji
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.applyPostponedSafeRule
{Q : Type}
[Queue Q]
(r : PostponedSafeRule)
(parentRef : GoalRef)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.runFirstUnsafeRule
{Q : Type}
[Queue Q]
(postponedSafeRules : Array PostponedSafeRule)
(parentRef : GoalRef)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
partial def
Aesop.runFirstUnsafeRule.loop
{Q : Type}
[Queue Q]
(parentRef : GoalRef)
(queue : UnsafeQueue)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.expandGoal.doUnsafe
{Q : Type}
[Queue Q]
(gref : GoalRef)
(postponedSafeRules : Array PostponedSafeRule)
:
Equations
- Aesop.expandGoal.doUnsafe gref postponedSafeRules = Aesop.withAesopTraceNode Aesop.TraceOption.steps Aesop.expandGoal.fmtUnsafe (Aesop.runFirstUnsafeRule postponedSafeRules gref)
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.expandGoal.fmtSafe
{Q : Type}
[Queue Q]
(result : Except Lean.Exception SafeRulesResult)
:
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.