src/HOLCF/Porder0.thy
changeset 3310 0ceaad3c3f52
parent 2850 a66196e1668c
child 3323 194ae2e0c193
--- a/src/HOLCF/Porder0.thy	Fri May 23 09:18:06 1997 +0200
+++ b/src/HOLCF/Porder0.thy	Fri May 23 09:20:35 1997 +0200
@@ -7,11 +7,11 @@
 
 *)
 
-Porder0 = Nat +
+Porder0 = Arith +
 
 (* first the global constant for HOLCF type classes *)
 consts
-  "less"        :: "['a,'a] => bool"
+  less        :: "['a,'a] => bool"
 
 axclass po < term
         (* class axioms: *)