(* Title: Example_Keyserver.thy Author: Andreas Viktor Hess, DTU SPDX-License-Identifier: BSD-3-Clause *) section ‹The Keyserver Example› theory Example_Keyserver imports "../Stateful_Compositionality" begin text ‹\label{sec:Example-Keyserver}› declare [[code_timing]] subsection ‹Setup› subsubsection ‹Datatypes and functions setup› datatype ex_lbl = Label1 (‹𝟭›) | Label2 (‹𝟮›)