equal
deleted
inserted
replaced
173 qed |
173 qed |
174 |
174 |
175 end %quote |
175 end %quote |
176 |
176 |
177 text {* |
177 text {* |
178 \noindent Note the occurence of the name @{text mult_nat} in the |
178 \noindent Note the occurrence of the name @{text mult_nat} in the |
179 primrec declaration; by default, the local name of a class operation |
179 primrec declaration; by default, the local name of a class operation |
180 @{text f} to be instantiated on type constructor @{text \<kappa>} is |
180 @{text f} to be instantiated on type constructor @{text \<kappa>} is |
181 mangled as @{text f_\<kappa>}. In case of uncertainty, these names may be |
181 mangled as @{text f_\<kappa>}. In case of uncertainty, these names may be |
182 inspected using the @{command "print_context"} command or the |
182 inspected using the @{command "print_context"} command or the |
183 corresponding ProofGeneral button. |
183 corresponding ProofGeneral button. |