diff -r 3b21b24a5fb6 -r a24e26f5488c Quot/Examples/AbsRepTest.thy --- a/Quot/Examples/AbsRepTest.thy Wed Dec 23 10:31:54 2009 +0100 +++ b/Quot/Examples/AbsRepTest.thy Wed Dec 23 13:23:33 2009 +0100 @@ -2,31 +2,12 @@ imports "../QuotMain" "../QuotList" "../QuotOption" "../QuotSum" "../QuotProd" List begin - -(* quotient_type fset = "'a list" / "\(xs::'a list) ys. \e. e \ set xs \ e \ set ys" apply(rule equivpI) unfolding reflp_def symp_def transp_def apply(auto) - sorry done -*) - -inductive - list_eq (infix "\" 50) -where - "a#b#xs \ b#a#xs" -| "[] \ []" -| "xs \ ys \ ys \ xs" -| "a#a#xs \ a#xs" -| "xs \ ys \ a#xs \ a#ys" -| "\xs1 \ xs2; xs2 \ xs3\ \ xs1 \ xs3" - -quotient_type - fset = "'a list" / "list_eq" - sorry - fun intrel :: "(nat \ nat) \ (nat \ nat) \ bool" @@ -36,7 +17,6 @@ quotient_type int = "nat \ nat" / intrel sorry - ML {* open Quotient_Term; *}