src/HOL/Quotient_Examples/Lift_RBT.thy
author kuncar
Tue, 31 Jul 2012 13:55:39 +0200
changeset 48622 caaa1a02c650
parent 48621 877df57629e3
permissions -rw-r--r--
use lifting/transfer formalization of RBT from Lift_RBT

(*  Title:      HOL/Quotient_Examples/Lift_RBT.thy
    Author:     Lukas Bulwahn and Ondrej Kuncar
*)

header {* Lifting operations of RBT trees *}

theory Lift_RBT 
imports Main "~~/src/HOL/Library/RBT_Impl"
begin

(* Moved to ~~/HOL/Library/RBT" *)

end