src/FOL/ex/If.ML
changeset 9205 f171fa6a0989
parent 5152 5b63f591678b
--- a/src/FOL/ex/If.ML	Thu Jun 29 22:39:57 2000 +0200
+++ b/src/FOL/ex/If.ML	Thu Jun 29 22:48:08 2000 +0200
@@ -1,12 +1,11 @@
-(*  Title:      FOL/ex/if
+(*  Title:      FOL/ex/If.ML
     ID:         $Id$
     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     Copyright   1991  University of Cambridge
 
-First-Order Logic: the 'if' example
+First-Order Logic: the 'if' example.
 *)
 
-open If;
 open Cla;    (*in case structure IntPr is open!*)
 
 val prems = Goalw [if_def]
@@ -42,7 +41,7 @@
 choplev 0;
 by (rewtac if_def);
 by (blast_tac FOL_cs 1);
-result();
+qed "";
 
 
 (*An invalid formula.  High-level rules permit a simpler diagnosis*)
@@ -58,7 +57,3 @@
 (*Check that subgoals remain: proof failed.*)
 getgoal 1; 
 by (REPEAT (step_tac FOL_cs 1));
-
-
-
-writeln"Reached end of file.";