src/HOL/Library/AList_Mapping.thy
changeset 58881 b9556a055632
parent 57850 34382a1f37d6
child 59487 adaa430fc0f7
equal deleted inserted replaced
58880:0baae4311a9f 58881:b9556a055632
     1 (* Title: HOL/Library/AList_Mapping.thy
     1 (* Title: HOL/Library/AList_Mapping.thy
     2    Author: Florian Haftmann, TU Muenchen
     2    Author: Florian Haftmann, TU Muenchen
     3 *)
     3 *)
     4 
     4 
     5 header {* Implementation of mappings with Association Lists *}
     5 section {* Implementation of mappings with Association Lists *}
     6 
     6 
     7 theory AList_Mapping
     7 theory AList_Mapping
     8 imports AList Mapping
     8 imports AList Mapping
     9 begin
     9 begin
    10 
    10