- rule : DisplayRuleName
- elapsed : Nanos
- successful : Bool
Instances For
Equations
Equations
Instances For
Equations
Equations
- Aesop.instToJsonRuleStats.toJson x✝ = Lean.Json.mkObj [[("rule", Lean.toJson x✝.rule)], [("elapsed", Lean.toJson x✝.elapsed)], [("successful", Lean.toJson x✝.successful)]].flatten
Instances For
Equations
- One or more equations did not get rendered due to their size.
Equations
Instances For
Equations
- One or more equations did not get rendered due to their size.
Equations
Instances For
Equations
Equations
Instances For
Equations
Equations
- Aesop.instInhabitedStats = { default := Aesop.instInhabitedStats.default }
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
Instances For
Equations
- Aesop.Stats.instEmptyCollection = { emptyCollection := Aesop.Stats.empty }
Equations
- Aesop.RuleStatsTotals.empty = { numSuccessful := 0, numFailed := 0, elapsedSuccessful := 0, elapsedFailed := 0 }
Instances For
Equations
- Aesop.RuleStatsTotals.instEmptyCollection = { emptyCollection := Aesop.RuleStatsTotals.empty }
Equations
- Aesop.RuleStatsTotals.compareByTotalElapsed = compareOn fun (totals : Aesop.RuleStatsTotals) => totals.elapsedSuccessful + totals.elapsedFailed
Instances For
def
Aesop.Stats.ruleStatsTotals
(p : Stats)
(init : Std.HashMap DisplayRuleName RuleStatsTotals := ∅)
:
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
@[reducible, inline]
Equations
Instances For
instance
Aesop.instMonadStatsStateRefT'
{m : Type → Type}
{ω σ : Type}
[MonadStats m]
:
MonadStats (StateRefT' ω σ m)
Equations
- One or more equations did not get rendered due to their size.
instance
Aesop.instMonadStatsReaderT
{m : Type → Type}
{α : Type}
[MonadStats m]
:
MonadStats (ReaderT α m)
Equations
- One or more equations did not get rendered due to their size.
instance
Aesop.instMonadStatsOfMonadOptionsOfMonadStateOfStats
{m : Type → Type}
[Lean.MonadOptions m]
[MonadStateOf Stats m]
:
Equations
- One or more equations did not get rendered due to their size.
@[always_inline]
Equations
- Aesop.enableStatsCollection = (fun (opts : Lean.Options) => Lean.Option.get opts Aesop.aesop.collectStats) <$> Lean.getOptions
Instances For
@[always_inline]
Instances For
@[always_inline]
Equations
- Aesop.enableStatsFile = do let __do_lift ← Lean.getOptions pure (Lean.Option.get __do_lift Aesop.aesop.stats.file != "")
Instances For
@[always_inline]
Equations
Instances For
@[always_inline]
def
Aesop.profiling
{m : Type → Type}
[Monad m]
[MonadStats m]
[MonadLiftT BaseIO m]
{α : Type}
(recordStats : Stats → α → Nanos → Stats)
(x : m α)
:
m α
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[always_inline]
def
Aesop.profilingRuleSelection
{m : Type → Type}
[Monad m]
[MonadStats m]
[MonadLiftT BaseIO m]
{α : Type}
:
m α → m α
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[always_inline]
def
Aesop.profilingRule
{m : Type → Type}
[Monad m]
[MonadStats m]
[MonadLiftT BaseIO m]
{α : Type}
(rule : DisplayRuleName)
(wasSuccessful : α → Bool)
:
m α → m α
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Aesop.modifyStatsIfEnabled
{m : Type → Type}
[Monad m]
[MonadStats m]
(f : Stats → Stats)
:
m Unit
Equations
- Aesop.modifyStatsIfEnabled f = do let __do_lift ← Aesop.enableStats if __do_lift = true then Aesop.modifyStats f else pure PUnit.unit
Instances For
def
Aesop.recordScriptGenerated
{m : Type → Type}
[Monad m]
[MonadStats m]
(x : ScriptGenerated)
:
m Unit
Equations
- One or more equations did not get rendered due to their size.