diff -r 54a3db2ed201 -r 903bb1495239 src/HOL/Library/Parallel.thy --- a/src/HOL/Library/Parallel.thy Wed Jun 17 10:57:11 2015 +0200 +++ b/src/HOL/Library/Parallel.thy Wed Jun 17 11:03:05 2015 +0200 @@ -1,12 +1,12 @@ (* Author: Florian Haftmann, TU Muenchen *) -section {* Futures and parallel lists for code generated towards Isabelle/ML *} +section \Futures and parallel lists for code generated towards Isabelle/ML\ theory Parallel imports Main begin -subsection {* Futures *} +subsection \Futures\ datatype 'a future = fork "unit \ 'a" @@ -26,7 +26,7 @@ code_reserved Eval Future future -subsection {* Parallel lists *} +subsection \Parallel lists\ definition map :: "('a \ 'b) \ 'a list \ 'b list" where [simp]: "map = List.map"