Documentation

Lean.PrettyPrinter

def Lean.PPContext.runCoreM {α : Type} (ppCtx : Lean.PPContext) (x : Lean.CoreM α) :
IO α
Equations
  • One or more equations did not get rendered due to their size.
Instances For
    def Lean.PPContext.runMetaM {α : Type} (ppCtx : Lean.PPContext) (x : Lean.MetaM α) :
    IO α
    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

          Return a fmt representing pretty-printed e together with a map from tags in fmt to Elab.Info nodes produced by the delaborator at various subexpressions of e.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            @[export lean_pp_expr]
            Equations
            • One or more equations did not get rendered due to their size.
            Instances For

              Pretty-prints a declaration c as c.{<levels>} <params> : <type>.

              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 Lean.MessageData.ofFormatWithInfos (fmt : Lean.MetaM Lean.FormatWithInfos) (noContext : optParam (UnitLean.Format) fun (x : Unit) => Std.Format.text "<no context, could not generate MessageData>") :

                  Turns a MetaM FormatWithInfos into a MessageData using .ofPPFormat and running the monadic value in the given context. Uses the pp.tagAppFns option to annotate constants with terminfo, which is necessary for seeing the type on mouse hover.

                  Equations
                  • One or more equations did not get rendered due to their size.
                  Instances For

                    Pretty print a const expression using delabConst and generate terminfo. This function avoids inserting @ if the constant is for a function whose first argument is implicit, which is what the default toMessageData for Expr does. Panics if e is not a constant.

                    Equations
                    • One or more equations did not get rendered due to their size.
                    Instances For

                      Generates MessageData for a declaration c as c.{<levels>} <params> : <type>, with terminfo.

                      Equations
                      Instances For