--- a/doc-src/TutorialI/Misc/simp.thy	Thu Dec 02 15:37:32 2010 +0100
+++ b/doc-src/TutorialI/Misc/simp.thy	Thu Dec 02 16:04:22 2010 +0100
@@ -422,7 +422,7 @@
 
 (*<*)lemma "x=x"
 (*>*)
-using [[trace_simp=true]]
+using [[simp_trace=true]]
 apply simp
 (*<*)oops(*>*)