diff -r 93c9022ba5e9 -r c4001cda9da3 Quot/Examples/FSet3.thy --- a/Quot/Examples/FSet3.thy Fri Feb 12 15:50:43 2010 +0100 +++ b/Quot/Examples/FSet3.thy Fri Feb 12 16:04:10 2010 +0100 @@ -136,7 +136,7 @@ quotient_definition "funion :: 'a fset \ 'a fset \ 'a fset" (infixl "|\|" 65) -as +is "op @" section {* Cardinality of finite sets *} @@ -227,12 +227,12 @@ quotient_definition "fmap :: ('a \ 'b) \ 'a fset \ 'b fset" -as +is "map" quotient_definition "fconcat :: ('a fset) fset => 'a fset" -as +is "concat" (*lemma fconcat_rsp[quot_respect]: @@ -619,19 +619,19 @@ quotient_definition "fdelete :: 'a fset \ 'a \ 'a fset" - as "delete_raw" + is "delete_raw" quotient_definition "finter :: 'a fset \ 'a fset \ 'a fset" ("_ \f _" [70, 71] 70) - as "inter_raw" + is "inter_raw" quotient_definition "ffold :: ('a \ 'b \ 'b) \ 'b \ 'a fset \ 'b" - as "fold_raw" + is "fold_raw" quotient_definition "fset_to_set :: 'a fset \ 'a set" - as "set" + is "set" section {* Lifted Theorems *} @@ -690,7 +690,7 @@ quotient_definition "fset_case :: 'a \ ('b \ 'b fset \ 'a) \ 'b fset \ 'a" -as +is "list_case" (* NOT SURE IF TRUE *)