doc-src/TutorialI/Misc/simp.thy
changeset 20143 54e493016486
parent 19792 e8e3da6d3ff7
child 20212 f4a8b4e2fb29
--- a/doc-src/TutorialI/Misc/simp.thy	Tue Jul 18 13:27:59 2006 +0200
+++ b/doc-src/TutorialI/Misc/simp.thy	Tue Jul 18 14:53:27 2006 +0200
@@ -483,7 +483,7 @@
 a theorem contains the name of the theory it comes from.
 
 Finallly, different search criteria can be combined arbitrarily. 
-The effect is conjuctive: Find returns the theorerms that satisfy all of
+The effect is conjuctive: Find returns the theorems that satisfy all of
 the criteria. For example,
 \begin{ttbox}
 "_ + _"  -"_ - _"  -simp: "_ * (_ + _)"  name: assoc