changeset 766 | df053507edba |
parent 705 | f51c6069cd17 |
child 767 | 37285ec4387d |
--- a/Quot/Examples/FSet2.thy Sun Dec 20 00:15:40 2009 +0100 +++ b/Quot/Examples/FSet2.thy Sun Dec 20 00:26:53 2009 +0100 @@ -21,7 +21,7 @@ unfolding equivp_reflp_symp_transp reflp_def symp_def transp_def by (auto intro: list_eq.intros list_eq_refl) -quotient fset = "'a list" / "list_eq" +quotient_type fset = "'a list" / "list_eq" by (rule equivp_list_eq) quotient_def