ProgTutorial/Intro.thy
changeset 529 13d7ea419c5f
parent 526 9e191bc4a828
child 530 aabb4c93a6ed
--- a/ProgTutorial/Intro.thy	Tue Jun 19 17:58:12 2012 +0100
+++ b/ProgTutorial/Intro.thy	Wed Jun 20 08:29:12 2012 +0100
@@ -288,15 +288,18 @@
   are by him.
 
   \item {\bf Lukas Bulwahn} made me aware of a problem with recursive
-  parsers and contributed exercise \ref{ex:contextfree} and contributed to
-  recipe \ref{rec:introspection}.
+  parsers and contributed exercise \ref{ex:contextfree} and contributed 
+  ``introspection'' of theorems 
+  \ref{sec:theorems}.
+
 
   \item {\bf Jeremy Dawson} wrote the first version of chapter \ref{chp:parsing}
   about parsing.
 
   \item {\bf Armin Heller} helped with recipe \ref{rec:sat}.
 
-  \item {\bf Rafal Kolanski} contributed to recipe \ref{rec:introspection}.
+  \item {\bf Rafal Kolanski} contributed the ``introspection'' of theorems 
+  \ref{sec:theorems}.
 
   \item {\bf Alexander Krauss} wrote a very early version of the ``first-steps'' 
   chapter and also contributed the material on @{ML_funct Named_Thms}.