aboutsummaryrefslogtreecommitdiffhomepage
path: root/printing/ppconstr.mli
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2017-07-24 21:01:23 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2017-08-29 05:18:49 +0200
commit5db048b7f9cb5d13e44d87a1007ff042eef25fb5 (patch)
treebf6904c27393270ca38b34d00b48968d99d5b023 /printing/ppconstr.mli
parent7a9205cd226c1df6a52afaee3374bc9cdffd6e8c (diff)
A new step of restructuration of notations.
This allows to issue a more appropriate message when a notation with a { } cannot be defined because of an incompatible level. E.g.: Notation "{ A } + B" := (sumbool A B) (at level 20).
Diffstat (limited to 'printing/ppconstr.mli')
-rw-r--r--printing/ppconstr.mli3
1 files changed, 2 insertions, 1 deletions
diff --git a/printing/ppconstr.mli b/printing/ppconstr.mli
index 833503485..7546c748d 100644
--- a/printing/ppconstr.mli
+++ b/printing/ppconstr.mli
@@ -15,6 +15,7 @@ open Libnames
open Constrexpr
open Names
open Misctypes
+open Notation_term
val extract_lam_binders :
constr_expr -> local_binder_expr list * constr_expr
@@ -24,7 +25,7 @@ val split_fix :
int -> constr_expr -> constr_expr ->
local_binder_expr list * constr_expr * constr_expr
-val prec_less : int -> int * Ppextend.parenRelation -> bool
+val prec_less : precedence -> tolerability -> bool
val pr_tight_coma : unit -> Pp.t