doc-src/TutorialI/Misc/simp.thy
changeset 36069 a15454b23ebd
parent 35992 78674c6018ca
child 40878 7695e4de4d86
--- a/doc-src/TutorialI/Misc/simp.thy	Sun Mar 28 19:34:08 2010 +0200
+++ b/doc-src/TutorialI/Misc/simp.thy	Mon Mar 29 09:47:21 2010 +0200
@@ -416,14 +416,20 @@
 In more complicated cases, the trace can be very lengthy.  Thus it is
 advisable to reset the \pgmenu{Trace Simplifier} flag after having
 obtained the desired trace.
-% Since this is easily forgotten (and may have the unpleasant effect of
-% swamping the interface with trace information), here is how you can switch
-% the trace on locally: * }
-%
-%using [[trace_simp=true]] apply(simp)
-% In fact, any proof step can be prefixed with this \isa{using} clause,
-% causing any local simplification to be traced.
- *}
+Since this is easily forgotten (and may have the unpleasant effect of
+swamping the interface with trace information), here is how you can switch
+the trace on locally in a proof: *}
+
+(*<*)lemma "x=x"
+(*>*)
+using [[trace_simp=true]]
+apply simp
+(*<*)oops(*>*)
+
+text{* \noindent
+Within the current proof, all simplifications in subsequent proof steps
+will be traced, but the text reminds you to remove the \isa{using} clause
+after it has done its job. *}
 
 subsection{*Finding Theorems\label{sec:find}*}