src/HOL/TLA/Buffer/Buffer.thy
changeset 41589 bbd861837ebc
parent 21624 6f79647cf536
child 58889 5b7a9633cfa8
equal deleted inserted replaced
41588:9546828c0eb3 41589:bbd861837ebc
     1 (*
     1 (*  Title:      HOL/TLA/Buffer/Buffer.thy
     2     File:        Buffer.thy
     2     Author:     Stephan Merz, University of Munich
     3     ID:          $Id$
       
     4     Author:      Stephan Merz
       
     5     Copyright:   1997 University of Munich
       
     6 *)
     3 *)
     7 
     4 
     8 header {* A simple FIFO buffer (synchronous communication, interleaving) *}
     5 header {* A simple FIFO buffer (synchronous communication, interleaving) *}
     9 
     6 
    10 theory Buffer
     7 theory Buffer