Equations
- Printf.errorShortFormat = "formatting string ended prematurely"
Instances For
Equations
- Printf.errorMissingArgument = "argument list ended prematurely"
Instances For
Equations
- Printf.errorBadArgument = "bad argument"
Instances For
- LeftAdjust : FormatAdjustment
- ZeroPad : FormatAdjustment
Instances For
Equations
- Printf.instReprFormatAdjustment = { reprPrec := Printf.reprFormatAdjustment✝ }
Equations
Equations
- Printf.instReprFormatSign = { reprPrec := Printf.reprFormatSign✝ }
Equations
- Printf.instInhabitedFormatSign = { default := Printf.FormatSign.Plus }
- adjust : Option FormatAdjustment
- sign : Option FormatSign
- alternate : Bool
- modifiers : String
- char : Char
Instances For
Equations
- Printf.instReprFieldFormat = { reprPrec := Printf.reprFieldFormat✝ }
Equations
- One or more equations did not get rendered due to their size.
@[reducible, inline]
Equations
Instances For
Equations
- Printf.instReprFormatParse = { reprPrec := Printf.reprFormatParse✝ }
@[reducible, inline]
Equations
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.
- Printf.vFmt c ufmt = ufmt
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.
- Printf.adjustSigned x✝¹ x✝ = Printf.adjust x✝¹ x✝
Instances For
Equations
- Printf.integral_prec none x✝ = x✝
- Printf.integral_prec (some 0) "0" = ""
- Printf.integral_prec (some prec) x✝ = "".pushn '0' (prec.toNat - x✝.length) ++ x✝
Instances For
def
Printf.showIntAtBase
{a : Type}
[OfNat a 0]
[OfNat a 1]
[Integral a]
[DecidableLT a]
[DecidableLE a]
[DecidableEq a]
:
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
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
- Printf.formatInt x✝¹ x✝ = Printf.formatIntegral (Printf.fixupMods x✝ none) (Printf.Integral.toInt x✝¹) x✝
Instances For
Equations
- Printf.formatChar x✝¹ x✝ = Printf.formatIntegral (some 0) (Printf.Integral.toInt x✝¹.toNat) (Printf.vFmt 'c' x✝)
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
- formatArg : a → FieldFormatter
- parseFormat : a → ModifierParser
Instances
Equations
- Printf.instPrintfArgChar = { formatArg := Printf.formatChar, parseFormat := fun (x : Char) (cf : String) => Printf.parseIntFormat 0 cf }
Equations
- Printf.instPrintfArgListOfIsChar = { formatArg := Printf.formatString }
Equations
- Printf.instPrintfArgString = { formatArg := Printf.formatString ∘ String.toList }
Equations
- Printf.instPrintfArgNat = { formatArg := Printf.formatInt, parseFormat := Printf.parseIntFormat }
Equations
- Printf.instPrintfArgInt = { formatArg := Printf.formatInt, parseFormat := Printf.parseIntFormat }
Equations
- Printf.instPrintfArgOfIntegralOfBounded = { formatArg := Printf.formatBoundedInt, parseFormat := Printf.parseIntFormat }
Equations
- Printf.instPrintfArgOfRealFloat = { formatArg := Printf.formatRealFloat }
@[reducible, inline]
Equations
Instances For
Equations
- One or more equations did not get rendered due to their size.
- Printf.getStar [] = Printf.perror✝ Printf.errorMissingArgument
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Printf.uprintf format us = Printf.uprintfs format.toList us ""