changeset 55837 | 154855d9a564 |
parent 54703 | 499f92dc6e45 |
child 56279 | b4d874f6c6be |
--- a/src/HOL/ex/ML.thy Sun Mar 02 18:41:41 2014 +0100 +++ b/src/HOL/ex/ML.thy Sun Mar 02 19:00:45 2014 +0100 @@ -104,7 +104,7 @@ *} text {* - The @{ML_struct Par_List} module provides high-level combinators for + The @{ML_structure Par_List} module provides high-level combinators for parallel list operations. *} ML {* timeit (fn () => map (fn n => ackermann 3 n) (1 upto 10)) *}