aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs
diff options
context:
space:
mode:
authorGravatar clrenard <clrenard@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-12-01 13:42:34 +0000
committerGravatar clrenard <clrenard@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-12-01 13:42:34 +0000
commit1d5d6427e6ab85f925207ee099729932c669ab16 (patch)
tree7e18c4f7a5ad373a3e6389d1a0da3129af00241f /proofs
parentac952fc310b1ba17c8e5a243ec617351130e1d81 (diff)
Amélioration du message d'erreur "w_unify"
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5051 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'proofs')
-rw-r--r--proofs/evar_refiner.ml10
1 files changed, 8 insertions, 2 deletions
diff --git a/proofs/evar_refiner.ml b/proofs/evar_refiner.ml
index 7ce48f2bb..2273ee760 100644
--- a/proofs/evar_refiner.ml
+++ b/proofs/evar_refiner.ml
@@ -24,6 +24,8 @@ open Proof_type
open Logic
open Refiner
open Tacexpr
+open Nameops
+
type wc = named_context sigma (* for a better reading of the following *)
@@ -106,8 +108,12 @@ let w_Define sp c wc =
let cty =
try
w_type_of (w_Focus sp wc) (mkCast (c,spdecl.evar_concl))
- with Not_found | (Type_errors.TypeError (_, Type_errors.UnboundVar _))->
- error "Instantiation contains unlegal variables"
+ with
+ Not_found -> error "Instantiation contains unlegal variables"
+ | (Type_errors.TypeError (e, Type_errors.UnboundVar v))->
+ errorlabstrm "w_Define"
+ (str "Cannot use variable " ++ pr_id v ++ str " to define " ++
+ str (string_of_existential sp))
in
match spdecl.evar_body with
| Evar_empty ->