aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2014-08-12 09:02:51 -0400
committerGravatar Pierre Boutillier <pierre.boutillier@pps.univ-paris-diderot.fr>2014-08-25 15:22:40 +0200
commit82312ad28ea14203cbfae9a7f69d2b8ab23c6b9f (patch)
tree4ad022401fdba8fdf94072c5dae77226d44de6f7
parentbc6e87572b33eb5d98cbb23522a71fd7d23931b7 (diff)
Grammar: "avoiding to" isn't proper, either
-rw-r--r--library/assumptions.ml2
-rw-r--r--pretyping/reductionops.ml2
-rw-r--r--test-suite/output/Arguments.out6
3 files changed, 5 insertions, 5 deletions
diff --git a/library/assumptions.ml b/library/assumptions.ml
index 37585caa4..e4638f5e4 100644
--- a/library/assumptions.ml
+++ b/library/assumptions.ml
@@ -187,7 +187,7 @@ let assumptions ?(add_opaque=false) ?(add_transparent=false) st (* t *) =
a "Let" definition, in the former it is an assumption of [t],
in the latter is must be unfolded like a Const.
The other cases are straightforward recursion.
- Calls to the environment are memoized, thus avoiding to explore
+ Calls to the environment are memoized, thus avoiding exploration of
the DAG of the environment as if it was a tree (can cause
exponential behavior and prevent the algorithm from terminating
in reasonable time). [s] is a set of [context_object], representing
diff --git a/pretyping/reductionops.ml b/pretyping/reductionops.ml
index 260a012aa..383066405 100644
--- a/pretyping/reductionops.ml
+++ b/pretyping/reductionops.ml
@@ -110,7 +110,7 @@ module ReductionBehaviour = struct
let never = List.mem `ReductionNeverUnfold flags in
let nomatch = List.mem `ReductionDontExposeCase flags in
let pp_nomatch = spc() ++ if nomatch then
- str "avoiding to expose match constructs" else str"" in
+ str "but avoid exposing match constructs" else str"" in
let pp_recargs = spc() ++ str "when the " ++
pr_enum (fun x -> pr_nth (x+1)) recargs ++ str (String.plural (List.length recargs) " argument") ++
str (String.plural (if List.length recargs >= 2 then 1 else 2) " evaluate") ++
diff --git a/test-suite/output/Arguments.out b/test-suite/output/Arguments.out
index dc421830f..629a1ab63 100644
--- a/test-suite/output/Arguments.out
+++ b/test-suite/output/Arguments.out
@@ -2,7 +2,7 @@ Nat.sub : nat -> nat -> nat
Nat.sub is not universe polymorphic
Argument scopes are [nat_scope nat_scope]
-The reduction tactics unfold Nat.sub avoiding to expose match constructs
+The reduction tactics unfold Nat.sub but avoid exposing match constructs
Nat.sub is transparent
Expands to: Constant Coq.Init.Nat.sub
Nat.sub : nat -> nat -> nat
@@ -10,7 +10,7 @@ Nat.sub : nat -> nat -> nat
Nat.sub is not universe polymorphic
Argument scopes are [nat_scope nat_scope]
The reduction tactics unfold Nat.sub when applied to 1 argument
- avoiding to expose match constructs
+ but avoid exposing match constructs
Nat.sub is transparent
Expands to: Constant Coq.Init.Nat.sub
Nat.sub : nat -> nat -> nat
@@ -19,7 +19,7 @@ Nat.sub is not universe polymorphic
Argument scopes are [nat_scope nat_scope]
The reduction tactics unfold Nat.sub
when the 1st argument evaluates to a constructor and
- when applied to 1 argument avoiding to expose match constructs
+ when applied to 1 argument but avoid exposing match constructs
Nat.sub is transparent
Expands to: Constant Coq.Init.Nat.sub
Nat.sub : nat -> nat -> nat