changeset 787 | 5cf83fa5b36c |
parent 768 | e9e205b904e2 |
child 833 | 129caba33c03 |
--- a/Quot/Examples/IntEx.thy Thu Dec 24 00:58:50 2009 +0100 +++ b/Quot/Examples/IntEx.thy Thu Dec 24 22:28:19 2009 +0100 @@ -7,7 +7,8 @@ where "intrel (x, y) (u, v) = (x + v = u + y)" -quotient_type my_int = "nat \<times> nat" / intrel +quotient_type + my_int = "nat \<times> nat" / intrel apply(unfold equivp_def) apply(auto simp add: mem_def expand_fun_eq) done