src/HOL/ex/CASC_Setup.thy
changeset 43161 27dcda8fc89b
parent 42827 8bfdcaf30551
child 43205 23b81469499f
--- a/src/HOL/ex/CASC_Setup.thy	Mon Jun 06 20:36:34 2011 +0200
+++ b/src/HOL/ex/CASC_Setup.thy	Mon Jun 06 20:36:34 2011 +0200
@@ -63,8 +63,8 @@
 *}
 
 method_setup isabellep = {*
-  Scan.lift Parse.nat >>
+  Scan.lift (Scan.optional Parse.nat 1) >>
     (fn m => fn ctxt => SIMPLE_METHOD (isabellep_tac ctxt m))
-*} ""
+*} "combination of Isabelle provers and oracles for CASC"
 
 end