author | bulwahn |
Wed, 14 Dec 2011 16:30:30 +0100 | |
changeset 45872 | 3759fb8a02b8 |
parent 45871 | 1fec5b365f9b |
child 45873 | 37ffb8797a63 |
--- a/src/HOL/Library/AList_Impl.thy Wed Dec 14 16:30:29 2011 +0100 +++ b/src/HOL/Library/AList_Impl.thy Wed Dec 14 16:30:30 2011 +0100 @@ -1,10 +1,10 @@ -(* Title: HOL/Library/AList.thy +(* Title: HOL/Library/AList_Impl.thy Author: Norbert Schirmer, Tobias Nipkow, Martin Wildmoser, TU Muenchen *) header {* Implementation of Association Lists *} -theory AList +theory AList_Impl imports Main More_List begin