changeset 766 | df053507edba |
parent 719 | a9e55e1ef64c |
child 767 | 37285ec4387d |
--- a/Quot/Examples/IntEx2.thy Sun Dec 20 00:15:40 2009 +0100 +++ b/Quot/Examples/IntEx2.thy Sun Dec 20 00:26:53 2009 +0100 @@ -11,7 +11,7 @@ where "intrel (x, y) (u, v) = (x + v = u + y)" -quotient int = "nat \<times> nat" / intrel +quotient_type int = "nat \<times> nat" / intrel unfolding equivp_def by (auto simp add: mem_def expand_fun_eq)