src/HOL/HoareParallel/Mul_Gar_Coll.thy
changeset 16417 9bc16273c2d4
parent 15247 98d3ca56684d
child 20050 a2fb9d553aad
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
     1 
     1 
     2 header {* \section{The Multi-Mutator Case} *}
     2 header {* \section{The Multi-Mutator Case} *}
     3 
     3 
     4 theory Mul_Gar_Coll = Graph + OG_Syntax:
     4 theory Mul_Gar_Coll imports Graph OG_Syntax begin
     5 
     5 
     6 text {*  The full theory takes aprox. 18 minutes.  *}
     6 text {*  The full theory takes aprox. 18 minutes.  *}
     7 
     7 
     8 record mut =
     8 record mut =
     9   Z :: bool
     9   Z :: bool