src/HOL/Library/Abstract_Rat.thy
changeset 42463 f270e3e18be5
parent 41528 276078f01ada
child 44779 98d597c4193d
--- a/src/HOL/Library/Abstract_Rat.thy	Fri Apr 22 15:57:43 2011 +0200
+++ b/src/HOL/Library/Abstract_Rat.thy	Sat Apr 23 13:00:19 2011 +0200
@@ -8,7 +8,7 @@
 imports Complex_Main
 begin
 
-types Num = "int \<times> int"
+type_synonym Num = "int \<times> int"
 
 abbreviation
   Num0_syn :: Num ("0\<^sub>N")