aboutsummaryrefslogtreecommitdiff
path: root/plugins
diff options
context:
space:
mode:
authorCyril Cohen2020-06-17 14:22:13 +0200
committerCyril Cohen2020-06-17 14:22:13 +0200
commit6499de1a834fa4e039246ac8b821ca23dd2a497e (patch)
tree0c0d418ecd8215f7850dea9dc8fefd1af93d6ba7 /plugins
parentfd173d59f79f3918ee5c3bd8b560b075a3749a75 (diff)
parent22ea81efe0111381be372d88821da8b2fa76be71 (diff)
Merge PR #12508: Fix #12507 Anomaly when using a ssreflect `reflect` view
Reviewed-by: CohenCyril Reviewed-by: ppedrot
Diffstat (limited to 'plugins')
-rw-r--r--plugins/ssr/ssrequality.ml12
1 files changed, 8 insertions, 4 deletions
diff --git a/plugins/ssr/ssrequality.ml b/plugins/ssr/ssrequality.ml
index 29a9c65561..da623703a2 100644
--- a/plugins/ssr/ssrequality.ml
+++ b/plugins/ssr/ssrequality.ml
@@ -389,17 +389,21 @@ let pirrel_rewrite ?(under=false) ?(map_redex=id_map_redex) pred rdx rdx_ty new_
ppdebug(lazy Pp.(str"pirrel_rewrite of type: " ++ pr_econstr_env env sigma proof_ty));
try Proofview.V82.of_tactic (refine_with
~first_goes_last:(not !ssroldreworder || under) ~with_evars:under (sigma, proof)) gl
- with _ ->
+ with e when CErrors.noncritical e ->
(* we generate a msg like: "Unable to find an instance for the variable" *)
let hd_ty, miss = match EConstr.kind sigma c with
| App (hd, args) ->
let hd_ty = Retyping.get_type_of env sigma hd in
- let names = let rec aux t = function 0 -> [] | n ->
+ let names = let rec aux env t = function 0 -> [] | n ->
let t = Reductionops.whd_all env sigma t in
let open EConstr in
match kind_of_type sigma t with
- | ProdType (name, _, t) -> name.binder_name :: aux t (n-1)
- | _ -> assert false in aux hd_ty (Array.length args) in
+ | ProdType (name, ty, t) ->
+ name.binder_name ::
+ aux (EConstr.push_rel (Context.Rel.Declaration.LocalAssum (name,ty)) env) t (n-1)
+ | _ ->
+ (* In the case the head is an HO constant it may accept more arguments *)
+ CList.init n (fun _ -> Names.Name.Anonymous) in aux env hd_ty (Array.length args) in
hd_ty, Util.List.map_filter (fun (t, name) ->
let evs = Evar.Set.elements (Evarutil.undefined_evars_of_term sigma t) in
let open_evs = List.filter (fun k ->