doc-src/IsarRef/Thy/Generic.thy
changeset 27092 3d79bbdaf2ef
parent 27071 614c045c5fd4
child 27209 388fd72e9f26
--- a/doc-src/IsarRef/Thy/Generic.thy	Sun Jun 08 14:29:36 2008 +0200
+++ b/doc-src/IsarRef/Thy/Generic.thy	Sun Jun 08 14:30:07 2008 +0200
@@ -375,7 +375,7 @@
     ('simp' | 'simp\_all') ('!' ?) opt? (simpmod *)
     ;
 
-    opt: '(' ('no\_asm' | 'no\_asm\_simp' | 'no\_asm\_use' | 'asm\_lr' | 'depth\_limit' ':' nat) ')'
+    opt: '(' ('no\_asm' | 'no\_asm\_simp' | 'no\_asm\_use' | 'asm\_lr' ) ')'
     ;
     simpmod: ('add' | 'del' | 'only' | 'cong' (() | 'add' | 'del') |
       'split' (() | 'add' | 'del')) ':' thmrefs
@@ -429,7 +429,7 @@
   for simplifying assumptions which are to the right of it (cf.\ @{ML
   asm_lr_simp_tac}).
 
-  Giving an option ``@{text "(depth_limit: n)"}'' limits the number of
+  The configuration option @{text "depth_limit"} limits the number of
   recursive invocations of the simplifier during conditional
   rewriting.