src/FOLP/IFOLP.thy
changeset 14854 61bdf2ae4dc5
parent 6509 9f7f4fd05b1f
child 17480 fd19f77dcf60
--- a/src/FOLP/IFOLP.thy	Tue Jun 01 11:25:26 2004 +0200
+++ b/src/FOLP/IFOLP.thy	Tue Jun 01 12:33:50 2004 +0200
@@ -10,17 +10,13 @@
 
 global
 
-classes term < logic
-
+classes term
 default term
 
 types
   p
   o
 
-arities
-  p,o :: logic
-
 consts  
       (*** Judgements ***)
  "@Proof"       ::   "[p,o]=>prop"      ("(_ /: _)" [51,10] 5)