src/Doc/Tutorial/Types/Axioms.thy
changeset 68484 59793df7f853
parent 67406 23307fd33906
child 69505 cc2d676d5395
equal deleted inserted replaced
68483:087d32a40129 68484:59793df7f853
   252 Table~\ref{tab:overloading} in the appendix.  Section
   252 Table~\ref{tab:overloading} in the appendix.  Section
   253 \ref{sec:numeric-classes} covers a range of corresponding classes
   253 \ref{sec:numeric-classes} covers a range of corresponding classes
   254 \emph{with} axioms.
   254 \emph{with} axioms.
   255 
   255 
   256 Further note that classes may contain axioms but \emph{no} operations.
   256 Further note that classes may contain axioms but \emph{no} operations.
   257 An example is class @{class finite} from theory @{theory Finite_Set}
   257 An example is class @{class finite} from theory @{theory "HOL.Finite_Set"}
   258 which specifies a type to be finite: @{lemma [source] "finite (UNIV :: 'a::finite
   258 which specifies a type to be finite: @{lemma [source] "finite (UNIV :: 'a::finite
   259 set)" by (fact finite_UNIV)}.\<close>
   259 set)" by (fact finite_UNIV)}.\<close>
   260 
   260 
   261 (*<*)end(*>*)
   261 (*<*)end(*>*)