aboutsummaryrefslogtreecommitdiffhomepage
path: root/vernac
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2018-04-12 16:09:04 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2018-04-12 16:09:04 +0200
commit1671fae4a020a66e329b9ea04c7e06aa13c71d1e (patch)
tree49085e71e3831ea16119362a4f87057e95c8f874 /vernac
parent8059a0efa79fcd72d56c424adf1bea10dae28d6d (diff)
Fixing the 3 cases of a "Stream.Error" ended with two periods.
The "Stream.Error" printer does add a period, so, the messages themselves should not.
Diffstat (limited to 'vernac')
-rw-r--r--vernac/comInductive.ml2
-rw-r--r--vernac/record.ml2
2 files changed, 2 insertions, 2 deletions
diff --git a/vernac/comInductive.ml b/vernac/comInductive.ml
index db2f16525..05c40dbdd 100644
--- a/vernac/comInductive.ml
+++ b/vernac/comInductive.ml
@@ -261,7 +261,7 @@ let check_param = function
| CLocalAssum (nas, Default _, _) -> List.iter check_named nas
| CLocalAssum (nas, Generalized _, _) -> ()
| CLocalPattern {CAst.loc} ->
- Loc.raise ?loc (Stream.Error "pattern with quote not allowed here.")
+ Loc.raise ?loc (Stream.Error "pattern with quote not allowed here")
let interp_mutual_inductive (paramsl,indl) notations cum poly prv finite =
check_all_names_different indl;
diff --git a/vernac/record.ml b/vernac/record.ml
index 6e745b2af..78e68e8a3 100644
--- a/vernac/record.ml
+++ b/vernac/record.ml
@@ -114,7 +114,7 @@ let typecheck_params_and_fields finite def id poly pl t ps nots fs =
(function CLocalDef (b, _, _) -> error default_binder_kind b
| CLocalAssum (ls, bk, ce) -> List.iter (error bk) ls
| CLocalPattern {CAst.loc} ->
- Loc.raise ?loc (Stream.Error "pattern with quote not allowed in record parameters.")) ps
+ Loc.raise ?loc (Stream.Error "pattern with quote not allowed in record parameters")) ps
in
let sigma, (impls_env, ((env1,newps), imps)) = interp_context_evars env0 sigma ps in
let sigma, typ, sort, template = match t with