| changeset 30663 | 0b6aff7451b2 |
| parent 30235 | 58d147683393 |
| child 32960 | 69916a850301 |
--- a/src/HOL/Library/AssocList.thy Mon Mar 23 08:14:23 2009 +0100 +++ b/src/HOL/Library/AssocList.thy Mon Mar 23 08:14:24 2009 +0100 @@ -1,12 +1,11 @@ (* Title: HOL/Library/AssocList.thy - ID: $Id$ Author: Norbert Schirmer, Tobias Nipkow, Martin Wildmoser *) header {* Map operations implemented on association lists*} theory AssocList -imports Plain "~~/src/HOL/Map" +imports Map Main begin text {*