changeset 787 | 5cf83fa5b36c |
parent 768 | e9e205b904e2 |
child 1128 | 17ca92ab4660 |
--- a/Quot/Examples/FSet2.thy Thu Dec 24 00:58:50 2009 +0100 +++ b/Quot/Examples/FSet2.thy Thu Dec 24 22:28:19 2009 +0100 @@ -21,7 +21,8 @@ unfolding equivp_reflp_symp_transp reflp_def symp_def transp_def by (auto intro: list_eq.intros list_eq_refl) -quotient_type fset = "'a list" / "list_eq" +quotient_type + 'a fset = "'a list" / "list_eq" by (rule equivp_list_eq) quotient_definition