src/Doc/Datatypes/Datatypes.thy
changeset 54616 a21a2223c02b
parent 54602 168790252038
child 54621 82a78bc9fa0d
equal deleted inserted replaced
54615:62fb5af93fe2 54616:a21a2223c02b
  2348 %    old \keyw{datatype}
  2348 %    old \keyw{datatype}
  2349 %
  2349 %
  2350 %  * @{command wrap_free_constructors}
  2350 %  * @{command wrap_free_constructors}
  2351 %    * @{text "no_discs_sels"}, @{text "rep_compat"}
  2351 %    * @{text "no_discs_sels"}, @{text "rep_compat"}
  2352 %    * hack to have both co and nonco view via locale (cf. ext nats)
  2352 %    * hack to have both co and nonco view via locale (cf. ext nats)
       
  2353 %  * code generator
       
  2354 %     * eq, refl, simps
  2353 *}
  2355 *}
  2354 
  2356 
  2355 
  2357 
  2356 (*
  2358 (*
  2357 subsection {* Introductory Example
  2359 subsection {* Introductory Example
  2381   ;
  2383   ;
  2382   X_list: '[' (X + ',') ']'
  2384   X_list: '[' (X + ',') ']'
  2383 "}
  2385 "}
  2384 
  2386 
  2385 % options: no_discs_sels rep_compat
  2387 % options: no_discs_sels rep_compat
  2386 
       
  2387 % X_list is as for BNF
       
  2388 
  2388 
  2389 \noindent
  2389 \noindent
  2390 Section~\ref{ssec:datatype-generated-theorems} lists the generated theorems.
  2390 Section~\ref{ssec:datatype-generated-theorems} lists the generated theorems.
  2391 *}
  2391 *}
  2392 
  2392