(* Title: HOL/Library/RBT_Impl.thy Author: Markus Reiter, TU Muenchen Author: Alexander Krauss, TU Muenchen *) section ‹Implementation of Red-Black Trees› theory RBT_Impl imports Main begin text ‹ For applications, you should use theory ‹RBT› which defines an abstract type of red-black tree obeying the invariant. › subsection ‹Datatype of RB trees› datatype color = R | B