src/HOL/Data_Structures/RBT.thy
changeset 61469 cd82b1023932
parent 61231 cc6969542f8d
child 61534 a88e07c8d0d5
--- a/src/HOL/Data_Structures/RBT.thy	Sat Oct 17 16:08:30 2015 +0200
+++ b/src/HOL/Data_Structures/RBT.thy	Sun Oct 18 17:25:13 2015 +0200
@@ -1,6 +1,6 @@
 (* Author: Tobias Nipkow *)
 
-section \<open>Red-Black Tree\<close>
+section \<open>Red-Black Trees\<close>
 
 theory RBT
 imports Tree2