ProgTutorial/Recipes/TimeLimit.thy
changeset 576 b78c4fab81a9
parent 569 f875a25aa72d
equal deleted inserted replaced
575:c3dbc04471a9 576:b78c4fab81a9
    39   programming on which @{ML \<open>apply\<close> in Timeout} relies.
    39   programming on which @{ML \<open>apply\<close> in Timeout} relies.
    40 
    40 
    41 \begin{readmore}
    41 \begin{readmore}
    42    The function @{ML \<open>apply\<close> in Timeout} is defined in the structure
    42    The function @{ML \<open>apply\<close> in Timeout} is defined in the structure
    43   @{ML_structure Timeout} which can be found in the file 
    43   @{ML_structure Timeout} which can be found in the file 
    44   @{ML_file "Pure/concurrent/timeout.ML"}.
    44   @{ML_file "Pure/Concurrent/timeout.ML"}.
    45 \end{readmore}
    45 \end{readmore}
    46 
    46 
    47  
    47  
    48 \<close>
    48 \<close>
    49 end
    49 end