src/Pure/General/base64.ML
author wenzelm
Mon, 02 Dec 2024 22:16:29 +0100
changeset 81541 5335b1ca6233
parent 76183 8089593a364a
permissions -rw-r--r--
more elementary operation Term.variant_bounds: only for bounds vs. frees, no consts, no tfrees;

(*  Title:      Pure/General/base64.ML
    Author:     Makarius

Support for Base64 data encoding (via Isabelle/Scala).
*)

signature BASE64 =
sig
  val decode: Bytes.T -> Bytes.T
  val encode: Bytes.T -> Bytes.T
end;

structure Base64: BASE64 =
struct

val decode = \<^scala>\<open>Base64.decode\<close>;
val encode = \<^scala>\<open>Base64.encode\<close>;

end;