src/HOL/Data_Structures/Tree23_Map.thy
changeset 62130 90a3016a6c12
parent 61790 0494964bb226
child 63411 e051eea34990
--- a/src/HOL/Data_Structures/Tree23_Map.thy	Mon Jan 11 18:27:27 2016 +0100
+++ b/src/HOL/Data_Structures/Tree23_Map.thy	Mon Jan 11 20:51:13 2016 +0100
@@ -1,6 +1,6 @@
 (* Author: Tobias Nipkow *)
 
-section \<open>A 2-3 Tree Implementation of Maps\<close>
+section \<open>2-3 Tree Implementation of Maps\<close>
 
 theory Tree23_Map
 imports