src/FOL/FOL.thy
changeset 5887 0864c6578d16
parent 4854 d1850e0964f2
child 7355 4c43090659ca
--- a/src/FOL/FOL.thy	Mon Nov 16 11:10:00 1998 +0100
+++ b/src/FOL/FOL.thy	Mon Nov 16 11:11:42 1998 +0100
@@ -4,7 +4,7 @@
 rules
   classical "(~P ==> P) ==> P"
 
-setup
-  ClasetThyData.setup
+setup ClasetThyData.setup
+setup attrib_setup              (* FIXME move to IFOL.thy *)
 
 end