src/HOL/HOLCF/Universal.thy
changeset 41295 5b5388d4ccc9
parent 41286 3d7685a4a5ff
child 41370 17b09240893c
--- a/src/HOL/HOLCF/Universal.thy	Sun Dec 19 18:10:54 2010 -0800
+++ b/src/HOL/HOLCF/Universal.thy	Sun Dec 19 18:11:20 2010 -0800
@@ -12,7 +12,7 @@
 
 subsubsection {* Basis datatype *}
 
-types ubasis = nat
+type_synonym ubasis = nat
 
 definition
   node :: "nat \<Rightarrow> ubasis \<Rightarrow> ubasis set \<Rightarrow> ubasis"