Documentation

Init.Data.Format.Basic

@[export lean_format_append]
Equations
Equations
Equations
class Std.Format.MonadPrettyFormat (m : TypeType) :
Type
  • pushOutput : Stringm Unit
  • pushNewline : Natm Unit
  • currColumn : m Nat
  • Start a scope tagged with n.

    startTag : Natm Unit
  • Exit the scope of n-many opened tags.

    endTags : Natm Unit

A monad in which we can pretty-print Format objects.

Instances
def Std.Format.prettyM {m : TypeType} (f : Lean.Format) (w : Nat) (indent : optParam Nat 0) [inst : Monad m] [inst : Std.Format.MonadPrettyFormat m] :
Equations
Equations
  • One or more equations did not get rendered due to their size.
@[export lean_format_pretty]

Pretty-print a Format object as a string with expected width w.

Equations
def Std.Format.joinSep {α : Type u} [inst : Lean.ToFormat α] :
Equations
def Std.Format.joinSuffix {α : Type u} [inst : Lean.ToFormat α] :
Equations