Documentation

Printf.Classes.PrintfArg

Equations
Instances For
    Equations
    Instances For
      Equations
      Instances For
        Equations
        Instances For
          def Printf.dfmt {f : Type u} [RealFloat f] (c : Char) (p? : Option Int) (alt : Bool) (x : f) :
          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            Instances For
              Instances For
                Instances For
                  Equations
                  • One or more equations did not get rendered due to their size.
                  @[reducible, inline]
                  Equations
                  Instances For

                    Walks over argument-type-specific modifier characters to find primary format character.

                    • modifiers : String

                      Modifiers found

                    • char : Char

                      Primary format character

                    • rest : String

                      Rest of the format string

                    Instances For
                      @[reducible, inline]
                      Equations
                      Instances For
                        def Printf.parseIntFormat {a : Sort u_1} :
                        a(s : String) → FormatParse
                        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
                              Instances For
                                Equations
                                Instances For
                                  Equations
                                  Instances For
                                    def Printf.showIntAtBase {a : Type} [OfNat a 0] [OfNat a 1] [Integral a] [DecidableLT a] [DecidableLE a] [DecidableEq a] :
                                    a(IntChar)aShowS
                                    Equations
                                    • One or more equations did not get rendered due to their size.
                                    Instances For
                                      partial def Printf.showIntAtBase.showIt {a : Type} [OfNat a 0] [Integral a] (base : a) (toChr : IntChar) :
                                      a × aStringString
                                      partial def Printf.fmtu.fmtu' (b : Int) :
                                      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
                                              def Printf.formatInt {a : Type u_1} [Integral a] :
                                              aFieldFormatShowS
                                              Equations
                                              Instances For
                                                Equations
                                                • One or more equations did not get rendered due to their size.
                                                Instances For
                                                  class Printf.PrintfArg (a : Type u) :
                                                  Instances
                                                    Equations
                                                    @[reducible, inline]
                                                    Equations
                                                    Instances For
                                                      Equations
                                                      Instances For
                                                        Equations
                                                        Instances For
                                                          Equations
                                                          • One or more equations did not get rendered due to their size.
                                                          Instances For
                                                            def Printf.uprintf (format : String) (us : List UPrintf) :
                                                            Equations
                                                            Instances For