aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar courtieu <courtieu@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-09-21 10:53:31 +0000
committerGravatar courtieu <courtieu@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-09-21 10:53:31 +0000
commitc92183a4bc227dbcfc3bf874801bd03724e5541d (patch)
tree505b6b855cee36579f04e3a39fefa50cf7ae365e
parent86002ce6e6fb3cbf1f5c9bf3657c13b4e79be192 (diff)
Report fix bug 2345 from v8.3 (Bad error message when functional
scheme was called on an unknown function anme). git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13445 85f007b7-540e-0410-9357-904b9bb8a0f7
-rw-r--r--plugins/funind/g_indfun.ml46
-rw-r--r--plugins/funind/indfun.ml4
2 files changed, 5 insertions, 5 deletions
diff --git a/plugins/funind/g_indfun.ml4 b/plugins/funind/g_indfun.ml4
index c97e79b23..200c52efc 100644
--- a/plugins/funind/g_indfun.ml4
+++ b/plugins/funind/g_indfun.ml4
@@ -187,7 +187,7 @@ let warning_error names e =
(str "Cannot define principle(s) for "++
h 1 (prlist_with_sep (fun _ -> str","++spc ()) Libnames.pr_reference names) ++
if do_observe () then Cerrors.explain_exn e else mt ())
- | _ -> anomaly ""
+ | _ -> raise e
VERNAC COMMAND EXTEND NewFunctionalScheme
@@ -215,11 +215,11 @@ VERNAC COMMAND EXTEND NewFunctionalScheme
end
| _ -> assert false (* we can only have non empty list *)
end
- | e ->
+ | e ->
let names = List.map (fun (_,na,_) -> na) fas in
warning_error names e
-
end
+
]
END
(***** debug only ***)
diff --git a/plugins/funind/indfun.ml b/plugins/funind/indfun.ml
index 346330b9a..9c3982cb5 100644
--- a/plugins/funind/indfun.ml
+++ b/plugins/funind/indfun.ml
@@ -274,7 +274,7 @@ let warning_error names e =
(str "Cannot define principle(s) for "++
h 1 (prlist_with_sep (fun _ -> str","++spc ()) Ppconstr.pr_id names) ++
e_explain e)
- | _ -> anomaly ""
+ | _ -> raise e
let error_error names e =
let e_explain e =
@@ -288,7 +288,7 @@ let error_error names e =
(str "Cannot define graph(s) for " ++
h 1 (prlist_with_sep (fun _ -> str","++spc ()) Ppconstr.pr_id names) ++
e_explain e)
- | _ -> anomaly ""
+ | _ -> raise e
let generate_principle on_error
is_general do_built (fix_rec_l:(Vernacexpr.fixpoint_expr * Vernacexpr.decl_notation list) list) recdefs interactive_proof