Quot/Examples/LarryInt.thy
changeset 766 df053507edba
parent 753 544b05e03ec0
child 767 37285ec4387d
--- a/Quot/Examples/LarryInt.thy	Sun Dec 20 00:15:40 2009 +0100
+++ b/Quot/Examples/LarryInt.thy	Sun Dec 20 00:26:53 2009 +0100
@@ -10,7 +10,7 @@
 where
   "intrel (x, y) (u, v) = (x + v = u + y)"
 
-quotient int = "nat \<times> nat" / intrel
+quotient_type int = "nat \<times> nat" / intrel
   by (auto simp add: equivp_def expand_fun_eq)
 
 instantiation int :: "{zero, one, plus, uminus, minus, times, ord}"