equal
deleted
inserted
replaced
2967 text {* |
2967 text {* |
2968 Plugins extend the (co)datatype package to interoperate with other Isabelle |
2968 Plugins extend the (co)datatype package to interoperate with other Isabelle |
2969 packages and tools, such as the code generator, Transfer, Lifting, and |
2969 packages and tools, such as the code generator, Transfer, Lifting, and |
2970 Quickcheck. They can be enabled or disabled individually using the |
2970 Quickcheck. They can be enabled or disabled individually using the |
2971 @{syntax plugins} option to the commands @{command datatype}, |
2971 @{syntax plugins} option to the commands @{command datatype}, |
2972 @{command codatatype}, @{command free_constructors}, @{command bnf}, and |
2972 @{command primrec}, @{command codatatype}, @{command primcorec}, |
2973 @{command bnf_axiomatization}. |
2973 @{command primcorecursive}, @{command bnf}, @{command bnf_axiomatization}, and |
2974 For example: |
2974 @{command free_constructors}. For example: |
2975 *} |
2975 *} |
2976 |
2976 |
2977 datatype (plugins del: code "quickcheck") color = Red | Black |
2977 datatype (plugins del: code "quickcheck") color = Red | Black |
2978 |
2978 |
2979 |
2979 |