src/FOL/IFOL.thy
changeset 4854 d1850e0964f2
parent 4793 03fd006fb97b
child 6027 9dd06eeda95c
--- a/src/FOL/IFOL.thy	Wed Apr 29 11:29:00 1998 +0200
+++ b/src/FOL/IFOL.thy	Wed Apr 29 11:29:39 1998 +0200
@@ -111,7 +111,8 @@
   eq_reflection   "(x=y)   ==> (x==y)"
   iff_reflection  "(P<->Q) ==> (P==Q)"
 
-end
 
+setup
+  Simplifier.setup
 
-ML val thy_setup = [Simplifier.setup];
+end