src/Doc/Codegen/Refinement.thy
changeset 53125 f4c6f8f6515b
parent 53015 a1119cf551e8
child 55422 6445a05a1234
equal deleted inserted replaced
53124:9ae9bbaccee1 53125:f4c6f8f6515b
   262 text %quotetypewriter {*
   262 text %quotetypewriter {*
   263   @{code_stmts Dlist.empty Dlist.insert Dlist.remove list_of_dlist (Haskell)}
   263   @{code_stmts Dlist.empty Dlist.insert Dlist.remove list_of_dlist (Haskell)}
   264 *}
   264 *}
   265 
   265 
   266 text {*
   266 text {*
       
   267   See further \cite{Haftmann-Kraus-Kuncar-Nipkow:2013:data_refinement}
       
   268   for the meta theory of datatype refinement involving invariants.
       
   269 
   267   Typical data structures implemented by representations involving
   270   Typical data structures implemented by representations involving
   268   invariants are available in the library, theory @{theory Mapping}
   271   invariants are available in the library, theory @{theory Mapping}
   269   specifies key-value-mappings (type @{typ "('a, 'b) mapping"});
   272   specifies key-value-mappings (type @{typ "('a, 'b) mapping"});
   270   these can be implemented by red-black-trees (theory @{theory RBT}).
   273   these can be implemented by red-black-trees (theory @{theory RBT}).
   271 *}
   274 *}