src/HOL/Refute.thy
changeset 17721 b943c01e1c6d
parent 16870 a1155e140597
child 21332 2605e1ccd9f2
--- a/src/HOL/Refute.thy	Thu Sep 29 15:50:43 2005 +0200
+++ b/src/HOL/Refute.thy	Thu Sep 29 15:50:44 2005 +0200
@@ -78,7 +78,7 @@
 (*                       This value is ignored under some ML compilers.      *)
 (* "satsolver"   string  Name of the SAT solver to be used.                  *)
 (*                                                                           *)
-(* See 'HOL/Main.thy' for default values.                                    *)
+(* See 'HOL/SAT.thy' for default values.                                     *)
 (*                                                                           *)
 (* The size of particular types can be specified in the form type=size       *)
 (* (where 'type' is a string, and 'size' is an int).  Examples:              *)
@@ -97,7 +97,7 @@
 (*                            syntax                                         *)
 (* HOL/Refute.thy             This file: loads the ML files, basic setup,    *)
 (*                            documentation                                  *)
-(* HOL/Main.thy               Sets default parameters                        *)
+(* HOL/SAT.thy                Sets default parameters                        *)
 (* HOL/ex/RefuteExamples.thy  Examples                                       *)
 (* ------------------------------------------------------------------------- *)
 \end{verbatim}