diff -r 08d9243bfaf1 -r ac1a14b5a085 doc-src/IsarAdvanced/Classes/Thy/Classes.thy --- a/doc-src/IsarAdvanced/Classes/Thy/Classes.thy Tue Dec 02 17:50:39 2008 +0100 +++ b/doc-src/IsarAdvanced/Classes/Thy/Classes.thy Wed Dec 03 09:51:35 2008 +0100 @@ -377,7 +377,7 @@ interpretation %quote idem_class: idem ["f \ (\\idem) \ \"] -by unfold_locales (rule idem) +proof qed (rule idem) text {* \noindent This gives you at hand the full power of the Isabelle module system; @@ -460,7 +460,7 @@ *} interpretation %quote list_monoid: monoid [append "[]"] - by unfold_locales auto + proof qed auto text {* \noindent This enables us to apply facts on monoids @@ -497,7 +497,7 @@ *} subclass %quote (in group) monoid -proof unfold_locales +proof fix x from invl have "x\
\ x = \" by simp with assoc [symmetric] neutl invl have "x\
\ (x \ \) = x\
\ x" by simp @@ -505,10 +505,8 @@ qed text {* - \noindent The logical proof is carried out on the locale level - and thus conveniently is opened using the @{text unfold_locales} - method which only leaves the logical differences still - open to proof to the user. Afterwards it is propagated + \noindent The logical proof is carried out on the locale level. + Afterwards it is propagated to the type system, making @{text group} an instance of @{text monoid} by adding an additional edge to the graph of subclass relations