aboutsummaryrefslogtreecommitdiffhomepage
path: root/intf
diff options
context:
space:
mode:
authorGravatar Gaëtan Gilbert <gaetan.gilbert@skyskimmer.net>2018-02-20 15:35:25 +0100
committerGravatar Gaëtan Gilbert <gaetan.gilbert@skyskimmer.net>2018-03-05 14:21:47 +0100
commit88f3b5a441a3aaeb637d0b109544fbe71b7560dd (patch)
treeddbe8c3c4e1e2d773078254b0cef162126503709 /intf
parent78551857a41a57607ecfb3fd010e0a9755f47cea (diff)
Allow universe declarations for [with Definition].
Diffstat (limited to 'intf')
-rw-r--r--intf/constrexpr.ml7
-rw-r--r--intf/vernacexpr.ml16
2 files changed, 17 insertions, 6 deletions
diff --git a/intf/constrexpr.ml b/intf/constrexpr.ml
index 5b51953bb..695c8fcb9 100644
--- a/intf/constrexpr.ml
+++ b/intf/constrexpr.ml
@@ -15,6 +15,11 @@ open Decl_kinds
(** [constr_expr] is the abstract syntax tree produced by the parser *)
+type universe_decl_expr = (lident list, glob_constraint list) gen_universe_decl
+
+type ident_decl = lident * universe_decl_expr option
+type name_decl = lname * universe_decl_expr option
+
type notation = string
type explicitation =
@@ -137,7 +142,7 @@ type constr_pattern_expr = constr_expr
type with_declaration_ast =
| CWith_Module of Id.t list Loc.located * qualid Loc.located
- | CWith_Definition of Id.t list Loc.located * constr_expr
+ | CWith_Definition of Id.t list Loc.located * universe_decl_expr option * constr_expr
type module_ast_r =
| CMident of qualid
diff --git a/intf/vernacexpr.ml b/intf/vernacexpr.ml
index ba28eacea..d81f4f0ba 100644
--- a/intf/vernacexpr.ml
+++ b/intf/vernacexpr.ml
@@ -158,11 +158,6 @@ type option_ref_value =
(** Identifier and optional list of bound universes and constraints. *)
-type universe_decl_expr = (lident list, glob_constraint list) gen_universe_decl
-
-type ident_decl = lident * universe_decl_expr option
-type name_decl = lname * universe_decl_expr option
-
type sort_expr = Sorts.family
type definition_expr =
@@ -534,3 +529,14 @@ type vernac_when =
| VtNow
| VtLater
type vernac_classification = vernac_type * vernac_when
+
+
+(** Deprecated stuff *)
+type universe_decl_expr = Constrexpr.universe_decl_expr
+[@@ocaml.deprecated "alias of Constrexpr.universe_decl_expr"]
+
+type ident_decl = Constrexpr.ident_decl
+[@@ocaml.deprecated "alias of Constrexpr.ident_decl"]
+
+type name_decl = Constrexpr.name_decl
+[@@ocaml.deprecated "alias of Constrexpr.name_decl"]