aboutsummaryrefslogtreecommitdiff
diff options
context:
space:
mode:
authorAbhishek Anand (optiplex7010@home)2020-02-22 13:22:27 -0800
committerHugo Herbelin2020-02-23 18:05:32 +0100
commit5820b274acda8be0372471758842b0ea2b950d41 (patch)
tree272a8c54fa449ff44c8bba215f4c021d5234d405
parentdd5a748cbec3abd9a11bbdd3ed4c14497b575fb9 (diff)
parens --> parentheses
-rw-r--r--interp/constrextern.ml2
-rw-r--r--interp/constrextern.mli2
-rw-r--r--printing/ppconstr.ml2
-rw-r--r--vernac/vernacentries.ml6
4 files changed, 6 insertions, 6 deletions
diff --git a/interp/constrextern.ml b/interp/constrextern.ml
index a5e7b89ded..bdfb63add3 100644
--- a/interp/constrextern.ml
+++ b/interp/constrextern.ml
@@ -59,7 +59,7 @@ let print_coercions = ref false
(* This forces printing of parentheses even when
it is implied by associativity/precedence *)
-let print_parens = ref false
+let print_parentheses = ref false
(* This forces printing universe names of Type{.} *)
let print_universes = Detyping.print_universes
diff --git a/interp/constrextern.mli b/interp/constrextern.mli
index 2691d27f69..0eca287c1d 100644
--- a/interp/constrextern.mli
+++ b/interp/constrextern.mli
@@ -53,7 +53,7 @@ val print_implicits_defensive : bool ref
val print_arguments : bool ref
val print_evar_arguments : bool ref
val print_coercions : bool ref
-val print_parens : bool ref
+val print_parentheses : bool ref
val print_universes : bool ref
val print_no_symbol : bool ref
val print_projections : bool ref
diff --git a/printing/ppconstr.ml b/printing/ppconstr.ml
index 6ede663883..d96a528b76 100644
--- a/printing/ppconstr.ml
+++ b/printing/ppconstr.ml
@@ -85,7 +85,7 @@ let tag_var = tag Tag.variable
let env = ref terms and envlist = ref termlists and bl = ref binders and bll = ref binderlists in
let pop r = let a = List.hd !r in r := List.tl !r; a in
let return unp pp1 pp2 = (tag_unparsing unp pp1) ++ pp2 in
- let parens = !Constrextern.print_parens in
+ let parens = !Constrextern.print_parentheses in
(* Warning:
The following function enforces a very precise order of
evaluation of sub-components.
diff --git a/vernac/vernacentries.ml b/vernac/vernacentries.ml
index cd8e699066..2eb1aa39b0 100644
--- a/vernac/vernacentries.ml
+++ b/vernac/vernacentries.ml
@@ -1282,9 +1282,9 @@ let () =
let () =
declare_bool_option
{ optdepr = false;
- optkey = ["Printing";"Parens"];
- optread = (fun () -> !Constrextern.print_parens);
- optwrite = (fun b -> Constrextern.print_parens := b) }
+ optkey = ["Printing";"Parentheses"];
+ optread = (fun () -> !Constrextern.print_parentheses);
+ optwrite = (fun b -> Constrextern.print_parentheses := b) }
let () =
declare_bool_option