diff options
| author | Gaëtan Gilbert | 2018-03-22 13:21:41 +0100 |
|---|---|---|
| committer | Gaëtan Gilbert | 2018-03-22 13:21:41 +0100 |
| commit | bca95952b541b209a3f8ca44d1ff119b976e54fb (patch) | |
| tree | cc4f6d8a466a0862a8fa3b4c0db8beef4a4c43c8 /intf | |
| parent | 9c5a447688365006c8e594edfb1e973db8d53454 (diff) | |
bool option -> (VernacCumulative | VernacNonCumulative) option
Diffstat (limited to 'intf')
| -rw-r--r-- | intf/vernacexpr.ml | 4 |
1 files changed, 2 insertions, 2 deletions
diff --git a/intf/vernacexpr.ml b/intf/vernacexpr.ml index df746f7653..c1c80b61d4 100644 --- a/intf/vernacexpr.ml +++ b/intf/vernacexpr.ml @@ -299,7 +299,7 @@ type module_binder = bool option * lident list * module_ast_inl (** [Some b] if locally enabled/disabled according to [b], [None] if we should use the global flag. *) -type cumulative_inductive_parsing_flag = bool option +type vernac_cumulative = VernacCumulative | VernacNonCumulative (** {6 The type of vernacular expressions} *) @@ -334,7 +334,7 @@ type nonrec vernac_expr = | VernacExactProof of constr_expr | VernacAssumption of (Decl_kinds.discharge * Decl_kinds.assumption_object_kind) * inline * (ident_decl list * constr_expr) with_coercion list - | VernacInductive of cumulative_inductive_parsing_flag * Decl_kinds.private_flag * inductive_flag * (inductive_expr * decl_notation list) list + | VernacInductive of vernac_cumulative option * Decl_kinds.private_flag * inductive_flag * (inductive_expr * decl_notation list) list | VernacFixpoint of Decl_kinds.discharge * (fixpoint_expr * decl_notation list) list | VernacCoFixpoint of Decl_kinds.discharge * (cofixpoint_expr * decl_notation list) list | VernacScheme of (lident option * scheme) list |
