src/Doc/Implementation/ML.thy
changeset 57417 29fe9bac501b
parent 57350 fc4d65afdf13
child 57421 94081154306d
equal deleted inserted replaced
57416:9188d901209d 57417:29fe9bac501b
  1933   @{assert} (a <> b);
  1933   @{assert} (a <> b);
  1934 *}
  1934 *}
  1935 
  1935 
  1936 text {* \medskip See @{file "~~/src/Pure/Concurrent/mailbox.ML"} how
  1936 text {* \medskip See @{file "~~/src/Pure/Concurrent/mailbox.ML"} how
  1937   to implement a mailbox as synchronized variable over a purely
  1937   to implement a mailbox as synchronized variable over a purely
  1938   functional queue. *}
  1938   functional list. *}
  1939 
  1939 
  1940 
  1940 
  1941 section {* Managed evaluation *}
  1941 section {* Managed evaluation *}
  1942 
  1942 
  1943 text {* Execution of Standard ML follows the model of strict
  1943 text {* Execution of Standard ML follows the model of strict