doc-src/TutorialI/Misc/types.thy
changeset 11457 279da0358aa9
parent 11456 7eb63f63e6c6
child 12327 5a4d78204492
equal deleted inserted replaced
11456:7eb63f63e6c6 11457:279da0358aa9
    26 text{*\noindent%
    26 text{*\noindent%
    27 Here \commdx{defs} is a keyword and
    27 Here \commdx{defs} is a keyword and
    28 @{thm[source]nand_def} and @{thm[source]xor_def} are user-supplied names.
    28 @{thm[source]nand_def} and @{thm[source]xor_def} are user-supplied names.
    29 The symbol \indexboldpos{\isasymequiv}{$IsaEq} is a special form of equality
    29 The symbol \indexboldpos{\isasymequiv}{$IsaEq} is a special form of equality
    30 that must be used in constant definitions.
    30 that must be used in constant definitions.
       
    31 Pattern-matching is not allowed: each definition must be of
       
    32 the form $f\,x@1\,\dots\,x@n~\isasymequiv~t$.
       
    33 Section~\ref{sec:Simp-with-Defs} explains how definitions are used
       
    34 in proofs.
       
    35 
    31 A \commdx{constdefs} command combines the effects of \isacommand{consts} and 
    36 A \commdx{constdefs} command combines the effects of \isacommand{consts} and 
    32 \isacommand{defs}.  For instance, we can introduce @{term"nand"} and @{term"xor"} by a 
    37 \isacommand{defs}.  For instance, we can introduce @{term"nand"} and @{term"xor"} by a 
    33 single command: 
    38 single command: 
    34 *}
    39 *}
    35 
    40