src/ZF/ex/CoUnit.thy
changeset 1401 0c439768f45c
parent 810 91c68f74f458
child 1478 2b8c2a7547ab
--- a/src/ZF/ex/CoUnit.thy	Fri Dec 08 19:48:15 1995 +0100
+++ b/src/ZF/ex/CoUnit.thy	Sat Dec 09 13:36:11 1995 +0100
@@ -17,7 +17,7 @@
   Coalgebra Theorem
 *)
 consts
-  counit :: "i"
+  counit :: i
 codatatype
   "counit" = Con ("x: counit")
 
@@ -27,7 +27,7 @@
 *)
 
 consts
-  counit2 :: "i"
+  counit2 :: i
 codatatype
   "counit2" = Con2 ("x: counit2", "y: counit2")