src/Doc/IsarRef/Generic.thy
changeset 50075 ceb877c315a1
parent 50071 959548c3b947
child 50076 c5cc24781cbf
--- a/src/Doc/IsarRef/Generic.thy	Wed Nov 07 16:45:33 2012 +0100
+++ b/src/Doc/IsarRef/Generic.thy	Wed Nov 07 21:43:02 2012 +0100
@@ -385,11 +385,17 @@
   simplification strategy, or incorporate other proof tools that solve
   sub-problems, produce rewrite rules on demand etc.
 
+  The rewriting strategy is always strictly bottom up, except for
+  congruence rules, which are applied while descending into a term.
+  Conditions in conditional rewrite rules are solved recursively
+  before the rewrite rule is applied.
+
   The default Simplifier setup of major object logics (HOL, HOLCF,
   FOL, ZF) makes the Simplifier ready for immediate use, without
   engaging into the internal structures.  Thus it serves as
   general-purpose proof tool with the main focus on equational
-  reasoning, and a bit more than that.  *}
+  reasoning, and a bit more than that.
+*}
 
 
 subsection {* Simplification methods \label{sec:simp-meth} *}