aboutsummaryrefslogtreecommitdiff
path: root/intf
diff options
context:
space:
mode:
authorEnrico Tassi2018-04-05 10:04:07 +0200
committerEnrico Tassi2018-04-05 10:04:07 +0200
commit4c3564ac7e2ea231a6dde84f2af6bfddbc0834c6 (patch)
treeba0f9bbbc04048c48a2128dde5bb89b2517e52c8 /intf
parentf97498a6c104da9b7b31f84505db76194a566f9b (diff)
parentbca95952b541b209a3f8ca44d1ff119b976e54fb (diff)
Merge PR #7016: Make parsing independent of the cumulativity flag.
Diffstat (limited to 'intf')
-rw-r--r--intf/vernacexpr.ml12
1 files changed, 4 insertions, 8 deletions
diff --git a/intf/vernacexpr.ml b/intf/vernacexpr.ml
index 76b35b08f1..06f969f19c 100644
--- a/intf/vernacexpr.ml
+++ b/intf/vernacexpr.ml
@@ -297,13 +297,9 @@ type inline =
type module_ast_inl = module_ast * inline
type module_binder = bool option * lident list * module_ast_inl
-(** Cumulativity can be set globally, locally or unset locally and it
- can not enabled at all. *)
-type cumulative_inductive_parsing_flag =
- | GlobalCumulativity
- | GlobalNonCumulativity
- | LocalCumulativity
- | LocalNonCumulativity
+(** [Some b] if locally enabled/disabled according to [b], [None] if
+ we should use the global flag. *)
+type vernac_cumulative = VernacCumulative | VernacNonCumulative
(** {6 The type of vernacular expressions} *)
@@ -338,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