src/FOLP/ex/foundn.ML
changeset 1464 a608f83e3421
parent 1459 d12da312eff4
child 3836 f1a1817659e6
--- a/src/FOLP/ex/foundn.ML	Tue Jan 30 15:12:53 1996 +0100
+++ b/src/FOLP/ex/foundn.ML	Tue Jan 30 15:19:20 1996 +0100
@@ -1,4 +1,4 @@
-(*  Title:      FOL/ex/foundn
+(*  Title:      FOLP/ex/foundn.ML
     ID:         $Id$
     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     Copyright   1991  University of Cambridge
@@ -6,7 +6,7 @@
 Intuitionistic FOL: Examples from The Foundation of a Generic Theorem Prover
 *)
 
-writeln"File FOL/ex/foundn.";
+writeln"File FOLP/ex/foundn.ML";
 
 goal IFOLP.thy "?p : A&B  --> (C-->A&C)";
 by (rtac impI 1);