diff -r cd2aca704279 -r c9f71476b030 Quotient-Paper/Paper.thy --- a/Quotient-Paper/Paper.thy Tue Oct 19 10:10:41 2010 +0100 +++ b/Quotient-Paper/Paper.thy Tue Oct 19 15:08:24 2010 +0100 @@ -28,12 +28,12 @@ fun_map ("_ \ _" 51) and fun_rel ("_ \ _" 51) and list_eq (infix "\" 50) and (* Not sure if we want this notation...? *) - fempty ("\") and - funion ("_ \ _") and - finsert ("{_} \ _") and + empty_fset ("\") and + union_fset ("_ \ _") and + insert_fset ("{_} \ _") and Cons ("_::_") and concat ("flat") and - fconcat ("\") and + concat_fset ("\") and Quotient ("Quot _ _ _") @@ -267,8 +267,8 @@ builds finite unions of finite sets: \begin{isabelle}\ \ \ \ \ %%% - @{thm fconcat_empty[THEN eq_reflection, no_vars]}\hspace{10mm} - @{thm fconcat_insert[THEN eq_reflection, no_vars]} + @{thm concat_empty_fset[THEN eq_reflection, no_vars]}\hspace{10mm} + @{thm concat_insert_fset[THEN eq_reflection, no_vars]} \end{isabelle} \noindent @@ -377,10 +377,13 @@ Using extensionality and unfolding the definition of @{text "\"}, we can get back to \eqref{adddef}. In what follows we shall use the convention to write @{text "map_\"} for a map-function - of the type-constructor @{text \}. For a type @{text \} with arguments @{text "\\<^isub>1\<^isub>\\<^isub>n"} the - type of the function @{text "map_\"} has to be @{text "\\<^isub>1\\\\\<^isub>n\\\<^isub>1\\\<^isub>n \"}. - For example @{text "map_list"} - has to have the type @{text "\\\ list"}. + of the type-constructor @{text \}. + %% a general type for map all types is difficult to give (algebraic types are + %% easy, but for example the function type is not algebraic + %For a type @{text \} with arguments @{text "\\<^isub>1\<^isub>\\<^isub>n"} the + %type of the function @{text "map_\"} has to be @{text "\\<^isub>1\\\\\<^isub>n\\\<^isub>1\\\<^isub>n \"}. + %For example @{text "map_list"} + %has to have the type @{text "\\\ list"}. In our implementation we maintain a database of these map-functions that can be dynamically extended.