Documentation

Lake.Toml.Elab.Value

TOML Value Elaboration #

Elaborates TOML values into Lean data types.

@[inline]
Equations
  • One or more equations did not get rendered due to their size.
Instances For
    def Lake.Toml.elabBoolean (x : Lean.TSyntax `Lake.Toml.boolean) :
    Equations
    • One or more equations did not get rendered due to their size.
    Instances For

      Numerals #

      Equations
      Instances For
        Equations
        Instances For
          def Lake.Toml.elabDecInt (x : Lean.TSyntax `Lake.Toml.decInt) :
          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.
              Instances For
                Equations
                • One or more equations did not get rendered due to their size.
                Instances For
                  def Lake.Toml.elabFloat (x : Lean.TSyntax `Lake.Toml.float) :
                  Equations
                  Instances For
                    def Lake.Toml.elabBinNum (x : Lean.TSyntax `Lake.Toml.binNum) :
                    Equations
                    • One or more equations did not get rendered due to their size.
                    Instances For
                      def Lake.Toml.elabOctNum (x : Lean.TSyntax `Lake.Toml.octNum) :
                      Equations
                      • One or more equations did not get rendered due to their size.
                      Instances For
                        Equations
                        Instances For
                          def Lake.Toml.elabHexNum (x : Lean.TSyntax `Lake.Toml.hexNum) :
                          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

                              Strings & Simple Keys #

                              def Lake.Toml.elabLiteralString (x : Lean.TSyntax `Lake.Toml.literalString) :
                              Equations
                              Instances For
                                def Lake.Toml.elabBasicString (x : Lean.TSyntax `Lake.Toml.basicString) :
                                Equations
                                Instances For
                                  Equations
                                  Instances For
                                    def Lake.Toml.elabMlLiteralString (x : Lean.TSyntax `Lake.Toml.mlLiteralString) :
                                    Equations
                                    Instances For
                                      def Lake.Toml.elabMlBasicString (x : Lean.TSyntax `Lake.Toml.mlBasicString) :
                                      Equations
                                      • One or more equations did not get rendered due to their size.
                                      Instances For
                                        def Lake.Toml.elabString (x : Lean.TSyntax `Lake.Toml.string) :
                                        Equations
                                        • One or more equations did not get rendered due to their size.
                                        Instances For
                                          @[inline]
                                          def Lake.Toml.elabUnquotedKey (x : Lean.TSyntax `Lake.Toml.unquotedKey) :
                                          Equations
                                          Instances For
                                            def Lake.Toml.elabSimpleKey (x : Lean.TSyntax `Lake.Toml.simpleKey) :
                                            Equations
                                            • One or more equations did not get rendered due to their size.
                                            Instances For

                                              Complex Values #

                                              def Lake.Toml.elabArray {α : Type} (x : Lean.TSyntax `Lake.Toml.array) (elabVal : Lean.TSyntax `Lake.Toml.valLean.CoreM α) :
                                              Equations
                                              • One or more equations did not get rendered due to their size.
                                              Instances For
                                                def Lake.Toml.elabInlineTable (x : Lean.TSyntax `Lake.Toml.inlineTable) (elabVal : Lean.TSyntax `Lake.Toml.valLean.CoreM Lake.Toml.Value) :
                                                Equations
                                                • One or more equations did not get rendered due to their size.
                                                Instances For