src/HOL/Data_Structures/RBT.thy
changeset 61231 cc6969542f8d
parent 61224 759b5299a9f2
child 61469 cd82b1023932
--- a/src/HOL/Data_Structures/RBT.thy	Tue Sep 22 17:13:13 2015 +0200
+++ b/src/HOL/Data_Structures/RBT.thy	Wed Sep 23 09:14:22 2015 +0200
@@ -1,6 +1,6 @@
 (* Author: Tobias Nipkow *)
 
-section \<open>Red-Black Trees\<close>
+section \<open>Red-Black Tree\<close>
 
 theory RBT
 imports Tree2