(* Title: HOL/ex/Tree23.thy Author: Tobias Nipkow, TU Muenchen *) section ‹2-3 Trees› theory Tree23 imports Main begin hide_const (open) or text‹This is a very direct translation of some of the functions in table.ML in the Isabelle source code. That source is due to Makarius Wenzel and Stefan Berghofer. Note that because of complicated patterns and mutual recursion, these function definitions take a few minutes and can also be seen as stress tests for the function definition facility.› type_synonym key = int ― ‹for simplicity, should be a type class›