doc-src/TutorialI/Inductive/Even.thy
changeset 23928 efee34ff4764
parent 23842 9d87177f1f89
child 25330 15bf0f47a87d
equal deleted inserted replaced
23927:cbe0e4aeb53c 23928:efee34ff4764
    14 *}
    14 *}
    15 
    15 
    16 subsection{* Making an Inductive Definition *}
    16 subsection{* Making an Inductive Definition *}
    17 
    17 
    18 text {*
    18 text {*
    19 Using \commdx{inductive\_set}, we declare the constant @{text even} to be
    19 Using \commdx{inductive\protect\_set}, we declare the constant @{text even} to be
    20 a set of natural numbers with the desired properties.
    20 a set of natural numbers with the desired properties.
    21 *}
    21 *}
    22 
    22 
    23 inductive_set even :: "nat set"
    23 inductive_set even :: "nat set"
    24 where
    24 where