Documentation

Lake.Util.Url

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    def Lake.uriEscapeByte (b : UInt8) (s : String := "") :

    Encode a byte as a URI escape code (e.g., %20).

    Equations
    Instances For
      @[specialize #[]]
      def Lake.foldlUtf8M {m : Type u_1 → Type u_2} {σ : Type u_1} [Monad m] (c : Char) (f : σUInt8m σ) (init : σ) :
      m σ

      Folds a monadic function over the UTF-8 bytes of Char from most significant to least significant.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        @[reducible, inline]
        abbrev Lake.foldlUtf8 {σ : Type u_1} (c : Char) (f : σUInt8σ) (init : σ) :
        σ
        Equations
        Instances For
          def Lake.uriEscapeChar (c : Char) (s : String := "") :

          Encode a character as a sequence of URI escape codes representing its UTF8 encoding.

          Equations
          Instances For

            A URI unreserved mark as specified in RFC3986. Unlike the older RFC2396, RFC2396 also reserves !, *, ', (, and ).

            Lake uses RFC3986 here because the curl implementation of AWS Sigv4 that Lake uses to upload artifacts requires these additional characters to be escaped.

            Equations
            Instances For
              def Lake.uriEncodeChar (c : Char) (s : String := "") :

              Encodes anything but a URI unreserved character as a URI escape sequences.

              Equations
              Instances For
                def Lake.uriEncode (s : String) (init : String := "") :

                Encodes a string as an ASCII URI component, escaping special characters (and unicode).

                Equations
                Instances For
                  def Lake.getUrl? (url : String) (headers : Array String := #[]) :

                  Performs a HTTP GET request of a URL (using curl with JSON output) and, if successful, return the body. Otherwise, returns none on a 404 and errors on anything else.

                  Equations
                  • One or more equations did not get rendered due to their size.
                  Instances For
                    def Lake.getUrl (url : String) (headers : Array String := #[]) :

                    Perform a HTTP GET request of a URL (using curl) and return the body.

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