src/Pure/General/zstd.ML
author Fabian Huch <huch@in.tum.de>
Thu, 16 Nov 2023 15:36:34 +0100
changeset 78980 a80ee3c97aae
parent 76351 2cee31cd92f0
permissions -rw-r--r--
properly concatenate toml files: regular toml rules still apply (e.g., inline values may not be changed), but values defined in one file may be updated in another;

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

Support for Zstd compression (via Isabelle/Scala).
*)

signature Zstd =
sig
  val compress: Bytes.T -> Bytes.T
  val uncompress: Bytes.T -> Bytes.T
end;

structure Zstd: Zstd =
struct

val compress = \<^scala>\<open>Zstd.compress\<close>;
val uncompress = \<^scala>\<open>Zstd.uncompress\<close>;

end;