src/HOL/Library/AList.thy
changeset 44913 48240fb48980
parent 44912 23956688856e
child 45605 a89b4bc311a5
--- a/src/HOL/Library/AList.thy	Tue Sep 13 09:25:19 2011 +0200
+++ b/src/HOL/Library/AList.thy	Tue Sep 13 09:28:03 2011 +0200
@@ -1,10 +1,10 @@
-(*  Title:      HOL/Library/AList_Impl.thy
+(*  Title:      HOL/Library/AList.thy
     Author:     Norbert Schirmer, Tobias Nipkow, Martin Wildmoser, TU Muenchen
 *)
 
 header {* Implementation of Association Lists *}
 
-theory AList_Impl 
+theory AList
 imports Main More_List
 begin