src/HOL/Map.thy
changeset 13914 026866537fae
parent 13912 3c0a340be514
child 13937 e9d57517c9b1
equal deleted inserted replaced
13913:b3ed67af04b8 13914:026866537fae
     3     Author:     Tobias Nipkow, based on a theory by David von Oheimb
     3     Author:     Tobias Nipkow, based on a theory by David von Oheimb
     4     Copyright   1997-2003 TU Muenchen
     4     Copyright   1997-2003 TU Muenchen
     5 
     5 
     6 The datatype of `maps' (written ~=>); strongly resembles maps in VDM.
     6 The datatype of `maps' (written ~=>); strongly resembles maps in VDM.
     7 *)
     7 *)
       
     8 
       
     9 header {* Maps *}
     8 
    10 
     9 theory Map = List:
    11 theory Map = List:
    10 
    12 
    11 types ('a,'b) "~=>" = "'a => 'b option" (infixr 0)
    13 types ('a,'b) "~=>" = "'a => 'b option" (infixr 0)
    12 
    14