changeset 58881 | b9556a055632 |
parent 57850 | 34382a1f37d6 |
child 59487 | adaa430fc0f7 |
--- a/src/HOL/Library/AList_Mapping.thy Sun Nov 02 17:16:01 2014 +0100 +++ b/src/HOL/Library/AList_Mapping.thy Sun Nov 02 17:20:45 2014 +0100 @@ -2,7 +2,7 @@ Author: Florian Haftmann, TU Muenchen *) -header {* Implementation of mappings with Association Lists *} +section {* Implementation of mappings with Association Lists *} theory AList_Mapping imports AList Mapping