src/Doc/Datatypes/Datatypes.thy
changeset 58659 6c9821c32dd5
parent 58620 7435b6a3f72e
child 58677 74a81d6f3c54
equal deleted inserted replaced
58658:9002fe021e2f 58659:6c9821c32dd5
   498 \begin{itemize}
   498 \begin{itemize}
   499 \setlength{\itemsep}{0pt}
   499 \setlength{\itemsep}{0pt}
   500 
   500 
   501 \item
   501 \item
   502 The @{text "plugins"} option indicates which plugins should be enabled
   502 The @{text "plugins"} option indicates which plugins should be enabled
   503 (@{text only}) or disabled (@{text del}). Wildcards (``@{text "*"}'') are
   503 (@{text only}) or disabled (@{text del}). Some plugin names are defined
   504 allowed (e.g., @{text "quickcheck_*"}). By default, all plugins are enabled.
   504 as indirection to a group of sub-plugins (notably @{text "quickcheck"}
       
   505 based on @{text quickcheck_random}, @{text quickcheck_exhaustive}, \dots).
       
   506 By default, all plugins are enabled.
   505 
   507 
   506 \item
   508 \item
   507 The @{text "discs_sels"} option indicates that discriminators and selectors
   509 The @{text "discs_sels"} option indicates that discriminators and selectors
   508 should be generated. The option is implicitly enabled if names are specified for
   510 should be generated. The option is implicitly enabled if names are specified for
   509 discriminators or selectors.
   511 discriminators or selectors.
  2792 @{command codatatype}, @{command free_constructors}, @{command bnf}, and
  2794 @{command codatatype}, @{command free_constructors}, @{command bnf}, and
  2793 @{command bnf_axiomatization}.
  2795 @{command bnf_axiomatization}.
  2794 For example:
  2796 For example:
  2795 *}
  2797 *}
  2796 
  2798 
  2797     datatype (plugins del: code "quickcheck_*") color = Red | Black
  2799     datatype (plugins del: code "quickcheck") color = Red | Black
  2798 
  2800 
  2799 
  2801 
  2800 subsection {* Code Generator
  2802 subsection {* Code Generator
  2801   \label{ssec:code-generator} *}
  2803   \label{ssec:code-generator} *}
  2802 
  2804