aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite
diff options
context:
space:
mode:
authorGravatar Benjamin Barenblat <bbaren@google.com>2018-07-22 18:19:26 -0400
committerGravatar Benjamin Barenblat <bbaren@google.com>2018-07-22 18:19:26 -0400
commit234f5479773d43a48e67c5c0ea361445c7fb6782 (patch)
tree0609f0aef4769561d3bee2049c5c973f40b20be3 /test-suite
parent32415df7e24d4d79a00fae95a5f619980b006c61 (diff)
Correct some spelling errorsmaster
Lintian found some spelling errors in the Debian packaging for coq. Fix them most places they appear in the current source. (Don't change documentation anchor names, as that would invalidate external deeplinks.) This also fixes a bug in coqdoc: prior to this commit, coqdoc would highlight `instanciate` but not `instantiate`.
Diffstat (limited to 'test-suite')
-rw-r--r--test-suite/bugs/closed/4132.v2
-rw-r--r--test-suite/success/univers.v2
2 files changed, 2 insertions, 2 deletions
diff --git a/test-suite/bugs/closed/4132.v b/test-suite/bugs/closed/4132.v
index 806ffb771..67ecc3087 100644
--- a/test-suite/bugs/closed/4132.v
+++ b/test-suite/bugs/closed/4132.v
@@ -26,6 +26,6 @@ Qed.
Lemma foo3 x y (b := 0) (H1 : x <= y) (H2 : y <= b) : x <= b.
omega. (* Pierre L: according to a comment of bug report #4132,
- this might have triggered "Failure(occurence 2)" in the past,
+ this might have triggered "Failure(occurrence 2)" in the past,
but I never managed to reproduce that. *)
Qed.
diff --git a/test-suite/success/univers.v b/test-suite/success/univers.v
index 286340459..28426b570 100644
--- a/test-suite/success/univers.v
+++ b/test-suite/success/univers.v
@@ -60,7 +60,7 @@ Qed.
Record U : Type := { A:=Type; a:A }.
-(** Check assignement of sorts to inductives and records. *)
+(** Check assignment of sorts to inductives and records. *)
Variable sh : list nat.