src/FOL/IFOL.thy
changeset 3906 5ae0e1324c56
parent 3835 9a5a4e123859
child 3932 436463f9f2b4
--- a/src/FOL/IFOL.thy	Thu Oct 16 15:31:12 1997 +0200
+++ b/src/FOL/IFOL.thy	Thu Oct 16 15:33:06 1997 +0200
@@ -8,6 +8,8 @@
 
 IFOL = Pure +
 
+global
+
 classes
   term < logic
 
@@ -62,6 +64,8 @@
   "op ~="       :: ['a, 'a] => o                (infixl "\\<noteq>" 50)
 
 
+path IFOL
+
 rules
 
   (* Equality *)
@@ -108,4 +112,3 @@
   iff_reflection  "(P<->Q) ==> (P==Q)"
 
 end
-