diff -r 206e2f1759cc -r 8fd9d555d04d doc-src/Classes/Thy/Classes.thy --- a/doc-src/Classes/Thy/Classes.thy Mon Feb 22 14:11:03 2010 +0100 +++ b/doc-src/Classes/Thy/Classes.thy Mon Feb 22 17:02:39 2010 +0100 @@ -362,17 +362,18 @@ text {* \noindent The connection to the type system is done by means - of a primitive axclass + of a primitive type class *} (*<*)setup %invisible {* Sign.add_path "foo" *} (*>*) -axclass %quote idem < type - idem: "f (f x) = f x" (*<*)setup %invisible {* Sign.parent_path *}(*>*) +classes %quote idem < type +(*<*)axiomatization where idem: "f (f (x::\\idem)) = f x" +setup %invisible {* Sign.parent_path *}(*>*) text {* \noindent together with a corresponding interpretation: *} interpretation %quote idem_class: idem "f \ (\\idem) \ \" -proof qed (rule idem) +(*<*)proof qed (rule idem)(*>*) text {* \noindent This gives you the full power of the Isabelle module system; @@ -414,8 +415,7 @@ subsection {* Derived definitions *} text {* - Isabelle locales support a concept of local definitions - in locales: + Isabelle locales are targets which support local definitions: *} primrec %quote (in monoid) pow_nat :: "nat \ \ \ \" where