(* Author: Matthias Brun, ETH Zürich, 2019 *) (* Author: Dmitriy Traytel, ETH Zürich, 2019 *) section ‹Syntax of $\lambda\bullet$› (*<*) theory Syntax imports Nominal2_Lemmas begin (*>*) typedecl hash instantiation hash :: pure begin definition permute_hash :: "perm ⇒ hash ⇒ hash" where "permute_hash π h = h" instance proof qed (simp_all add: permute_hash_def) end atom_decl var