src/Doc/Datatypes/Datatypes.thy
changeset 52868 cca9e958da5c
parent 52843 ea95702328cf
child 52969 f2df0730f8ac
equal deleted inserted replaced
52867:8d8cb75ab20a 52868:cca9e958da5c
   218 *}
   218 *}
   219 
   219 
   220     datatype_new nat = Zero | Suc nat
   220     datatype_new nat = Zero | Suc nat
   221 
   221 
   222 text {*
   222 text {*
   223 Setup to be able to write @{term 0} instead of @{const Zero}:
   223 Setup to be able to write @{text 0} instead of @{const Zero}:
   224 *}
   224 *}
   225 
   225 
   226     instantiation nat :: zero
   226     instantiation nat :: zero
   227     begin
   227     begin
   228     definition "0 = Zero"
   228     definition "0 = Zero"