def
Aesop.Goal.withHeadlineTraceNode
{α : Type}
(g : Goal)
(traceOpt : TraceOption)
(k : Lean.MetaM α)
(collapsed : Bool := true)
(transform : Lean.MessageData → Lean.MetaM Lean.MessageData := pure)
:
Equations
- g.withHeadlineTraceNode traceOpt k collapsed transform = Aesop.withConstAesopTraceNode traceOpt (Aesop.Goal.withHeadlineTraceNode.fmt g transform) k collapsed
Instances For
def
Aesop.Goal.withHeadlineTraceNode.fmt
(g : Goal)
(transform : Lean.MessageData → Lean.MetaM Lean.MessageData := pure)
:
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.Goal.traceMetadata.trc traceOpt msg = Lean.addTrace traceOpt.traceClass (Lean.toMessageData msg)
Instances For
def
Aesop.Goal.traceMetadata.trcNode
(traceOpt : TraceOption)
(msg : Lean.MessageData)
(k : Lean.MetaM Unit)
:
Equations
- Aesop.Goal.traceMetadata.trcNode traceOpt msg k = Aesop.withConstAesopTraceNode traceOpt (pure msg) k
Instances For
def
Aesop.Rapp.withHeadlineTraceNode
{α : Type}
(r : Rapp)
(traceOpt : TraceOption)
(k : Lean.MetaM α)
(collapsed : Bool := true)
(transform : Lean.MessageData → Lean.MetaM Lean.MessageData := pure)
:
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.Rapp.traceMetadata.trc traceOpt m = Lean.addTrace traceOpt.traceClass (Lean.toMessageData m)