aboutsummaryrefslogtreecommitdiff
path: root/pretyping
diff options
context:
space:
mode:
authorEnrico Tassi2020-07-10 19:19:30 +0200
committerEnrico Tassi2020-07-10 19:19:30 +0200
commit7e149d3e7c7c6690b6aa92887d28e42f997b148a (patch)
treecea5ab4b0310188c384a0afd03fc15cdf98bcf06 /pretyping
parent511d2caaffb8d412d1645f0a83c9b0a2bbc41411 (diff)
parent9065877add52fa94de699ee8a50d240fb7ef4a5c (diff)
Merge PR #12638: Some changes of representation in Tacred
Ack-by: backtracking Reviewed-by: gares
Diffstat (limited to 'pretyping')
-rw-r--r--pretyping/reductionops.ml14
-rw-r--r--pretyping/reductionops.mli26
-rw-r--r--pretyping/tacred.ml282
3 files changed, 154 insertions, 168 deletions
diff --git a/pretyping/reductionops.ml b/pretyping/reductionops.ml
index 6f02d76f3a..594b8ab54c 100644
--- a/pretyping/reductionops.ml
+++ b/pretyping/reductionops.ml
@@ -436,15 +436,11 @@ type state = constr * constr Stack.t
type reduction_function = env -> evar_map -> constr -> constr
type e_reduction_function = env -> evar_map -> constr -> evar_map * constr
-type contextual_stack_reduction_function =
+type stack_reduction_function =
env -> evar_map -> constr -> constr * constr list
-type stack_reduction_function = contextual_stack_reduction_function
-type local_stack_reduction_function =
- evar_map -> constr -> constr * constr list
type state_reduction_function =
env -> evar_map -> state -> state
-type local_state_reduction_function = evar_map -> state -> state
let pr_state env sigma (tm,sk) =
let open Pp in
@@ -572,14 +568,6 @@ let reduce_and_refold_fix recfun env sigma fix sk =
(fun _ (t,sk') -> recfun (t,sk'))
[] sigma raw_answer sk
-let fix_recarg ((recindices,bodynum),_) stack =
- assert (0 <= bodynum && bodynum < Array.length recindices);
- let recargnum = Array.get recindices bodynum in
- try
- Some (recargnum, Stack.nth stack recargnum)
- with Not_found ->
- None
-
open Primred
module CNativeEntries =
diff --git a/pretyping/reductionops.mli b/pretyping/reductionops.mli
index b316b3c213..218936edfb 100644
--- a/pretyping/reductionops.mli
+++ b/pretyping/reductionops.mli
@@ -112,15 +112,11 @@ type reduction_function = env -> evar_map -> constr -> constr
type e_reduction_function = env -> evar_map -> constr -> evar_map * constr
-type contextual_stack_reduction_function =
+type stack_reduction_function =
env -> evar_map -> constr -> constr * constr list
-type stack_reduction_function = contextual_stack_reduction_function
-type local_stack_reduction_function =
- evar_map -> constr -> constr * constr list
type state_reduction_function =
env -> evar_map -> state -> state
-type local_state_reduction_function = evar_map -> state -> state
val pr_state : env -> evar_map -> state -> Pp.t
@@ -130,11 +126,6 @@ val strong_with_flags :
(CClosure.RedFlags.reds -> reduction_function) ->
(CClosure.RedFlags.reds -> reduction_function)
val strong : reduction_function -> reduction_function
-(*i
-val stack_reduction_of_reduction :
- 'a reduction_function -> 'a state_reduction_function
-i*)
-val stacklam : (state -> 'a) -> constr list -> evar_map -> constr -> constr Stack.t -> 'a
val whd_state_gen :
CClosure.RedFlags.reds -> Environ.env -> Evd.evar_map -> state -> state
@@ -167,13 +158,13 @@ val whd_allnolet : reduction_function
val whd_betalet : reduction_function
(** Removes cast and put into applicative form *)
-val whd_nored_stack : contextual_stack_reduction_function
-val whd_beta_stack : contextual_stack_reduction_function
-val whd_betaiota_stack : contextual_stack_reduction_function
-val whd_betaiotazeta_stack : contextual_stack_reduction_function
-val whd_all_stack : contextual_stack_reduction_function
-val whd_allnolet_stack : contextual_stack_reduction_function
-val whd_betalet_stack : contextual_stack_reduction_function
+val whd_nored_stack : stack_reduction_function
+val whd_beta_stack : stack_reduction_function
+val whd_betaiota_stack : stack_reduction_function
+val whd_betaiotazeta_stack : stack_reduction_function
+val whd_all_stack : stack_reduction_function
+val whd_allnolet_stack : stack_reduction_function
+val whd_betalet_stack : stack_reduction_function
val whd_nored_state : state_reduction_function
val whd_beta_state : state_reduction_function
@@ -242,7 +233,6 @@ val is_arity : env -> evar_map -> constr -> bool
val is_sort : env -> evar_map -> types -> bool
val contract_fix : evar_map -> fixpoint -> constr
-val fix_recarg : ('a, 'a) pfixpoint -> 'b Stack.t -> (int * 'b) option
(** {6 Querying the kernel conversion oracle: opaque/transparent constants } *)
val is_transparent : Environ.env -> Constant.t tableKey -> bool
diff --git a/pretyping/tacred.ml b/pretyping/tacred.ml
index baa32565f6..e4b5dc1edf 100644
--- a/pretyping/tacred.ml
+++ b/pretyping/tacred.ml
@@ -358,30 +358,6 @@ let reference_eval env sigma = function
let x = Name default_dependent_ident
-let make_elim_fun (names,(nbfix,lv,n)) u largs =
- let lu = List.firstn n largs in
- let p = List.length lv in
- let lyi = List.map fst lv in
- let la =
- List.map_i (fun q aq ->
- (* k from the comment is q+1 *)
- try mkRel (p+1-(List.index Int.equal (n-q) lyi))
- with Not_found -> aq)
- 0 (List.map (Vars.lift p) lu)
- in
- fun i ->
- match names.(i) with
- | None -> None
- | Some (minargs,ref) ->
- let body = applist (mkEvalRef ref u, la) in
- let g =
- List.fold_left_i (fun q (* j = n+1-q *) c (ij,tij) ->
- let subst = List.map (Vars.lift (-q)) (List.firstn (n-ij) la) in
- let tij' = Vars.substl (List.rev subst) tij in
- let x = make_annot x Sorts.Relevant in (* TODO relevance *)
- mkLambda (x,tij',c)) 1 body (List.rev lv)
- in Some (minargs,g)
-
(* [f] is convertible to [Fix(recindices,bodynum),bodyvect)]:
do so that the reduction uses this extra information *)
@@ -467,16 +443,6 @@ let substl_checking_arity env subst sigma c =
type fix_reduction_result = NotReducible | Reduced of (constr * constr list)
-let reduce_fix whdfun sigma fix stack =
- match fix_recarg fix (Stack.append_app_list stack Stack.empty) with
- | None -> NotReducible
- | Some (recargnum,recarg) ->
- let (recarg'hd,_ as recarg') = whdfun sigma recarg in
- let stack' = List.assign stack recargnum (applist recarg') in
- (match EConstr.kind sigma recarg'hd with
- | Construct _ -> Reduced (contract_fix sigma fix, stack')
- | _ -> NotReducible)
-
let contract_fix_use_function env sigma f
((recindices,bodynum),(_names,_types,bodies as typedbodies)) =
let nbodies = Array.length recindices in
@@ -484,22 +450,6 @@ let contract_fix_use_function env sigma f
let lbodies = List.init nbodies make_Fi in
substl_checking_arity env (List.rev lbodies) sigma (nf_beta env sigma bodies.(bodynum))
-let reduce_fix_use_function env sigma f whfun fix stack =
- match fix_recarg fix (Stack.append_app_list stack Stack.empty) with
- | None -> NotReducible
- | Some (recargnum,recarg) ->
- let (recarg'hd,_ as recarg') =
- if EConstr.isRel sigma recarg then
- (* The recarg cannot be a local def, no worry about the right env *)
- (recarg, [])
- else
- whfun recarg in
- let stack' = List.assign stack recargnum (applist recarg') in
- (match EConstr.kind sigma recarg'hd with
- | Construct _ ->
- Reduced (contract_fix_use_function env sigma f fix,stack')
- | _ -> NotReducible)
-
let contract_cofix_use_function env sigma f
(bodynum,(_names,_,bodies as typedbodies)) =
let nbodies = Array.length bodies in
@@ -574,34 +524,23 @@ let match_eval_ref_value env sigma constr stack =
env |> lookup_rel n |> RelDecl.get_value |> Option.map (lift n)
| _ -> None
-let special_red_case env sigma whfun (ci, p, iv, c, lf) =
- let rec redrec s =
- let (constr, cargs) = whfun s in
- match match_eval_ref env sigma constr cargs with
- | Some (ref, u) ->
- (match reference_opt_value env sigma ref u with
- | None -> raise Redelimination
- | Some gvalue ->
- if reducible_mind_case sigma gvalue then
- reduce_mind_case_use_function constr env sigma
- {mP=p; mconstr=gvalue; mcargs=cargs;
- mci=ci; mlf=lf}
- else
- redrec (applist(gvalue, cargs)))
- | None ->
- if reducible_mind_case sigma constr then
- reduce_mind_case sigma
- {mP=p; mconstr=constr; mcargs=cargs;
- mci=ci; mlf=lf}
- else
- raise Redelimination
- in
- redrec c
+let push_app sigma (hd, stk as p) = match EConstr.kind sigma hd with
+| App (hd, args) ->
+ (hd, Array.fold_right (fun x accu -> x :: accu) args stk)
+| _ -> p
let recargs = function
| EvalVar _ | EvalRel _ | EvalEvar _ -> None
| EvalConst c -> ReductionBehaviour.get (GlobRef.ConstRef c)
+let fix_recarg ((recindices,bodynum),_) stack =
+ assert (0 <= bodynum && bodynum < Array.length recindices);
+ let recargnum = Array.get recindices bodynum in
+ try
+ Some (recargnum, List.nth stack recargnum)
+ with Failure _ ->
+ None
+
let reduce_projection env sigma p ~npars (recarg'hd,stack') stack =
(match EConstr.kind sigma recarg'hd with
| Construct _ ->
@@ -609,24 +548,9 @@ let reduce_projection env sigma p ~npars (recarg'hd,stack') stack =
Reduced (List.nth stack' proj_narg, stack)
| _ -> NotReducible)
-let reduce_proj env sigma whfun whfun' c =
- let rec redrec s =
- match EConstr.kind sigma s with
- | Proj (proj, c) ->
- let c' = try redrec c with Redelimination -> c in
- let constr, cargs = whfun c' in
- (match EConstr.kind sigma constr with
- | Construct _ ->
- let proj_narg = Projection.npars proj + Projection.arg proj in
- List.nth cargs proj_narg
- | _ -> raise Redelimination)
- | Case (n,p,iv,c,brs) ->
- let c' = redrec c in
- let p = (n,p,iv,c',brs) in
- (try special_red_case env sigma whfun' p
- with Redelimination -> mkCase p)
- | _ -> raise Redelimination
- in redrec c
+let rec beta_applist sigma accu c stk = match EConstr.kind sigma c, stk with
+| Lambda (_, _, c), arg :: stk -> beta_applist sigma (arg :: accu) c stk
+| _ -> substl accu c, stk
let whd_nothing_for_iota env sigma s =
let rec whrec (x, stack as s) =
@@ -650,17 +574,17 @@ let whd_nothing_for_iota env sigma s =
(match constant_opt_value_in env (const, u) with
| Some body -> whrec (EConstr.of_constr body, stack)
| None -> s)
- | LetIn (_,b,_,c) -> stacklam whrec [b] sigma c stack
+ | LetIn (_,b,_,c) -> whrec (beta_applist sigma [b] c stack)
| Cast (c,_,_) -> whrec (c, stack)
- | App (f,cl) -> whrec (f, Stack.append_app cl stack)
+ | App (f,cl) -> whrec (f, Array.fold_right (fun c accu -> c :: accu) cl stack)
| Lambda (na,t,c) ->
- (match Stack.decomp stack with
- | Some (a,m) -> stacklam whrec [a] sigma c m
+ (match stack with
+ | a :: stack -> whrec (beta_applist sigma [a] c stack)
| _ -> s)
| x -> s
in
- EConstr.decompose_app sigma (Stack.zip sigma (whrec (s,Stack.empty)))
+ whrec s
(* [red_elim_const] contracts iota/fix/cofix redexes hidden behind
constants by keeping the name of the constants in the recursive calls;
@@ -703,21 +627,17 @@ let rec red_elim_const env sigma ref u largs =
try match reference_eval env sigma ref with
| EliminationCases n when nargs >= n ->
let c = reference_value env sigma ref u in
- let c', lrest = whd_nothing_for_iota env sigma (applist(c,largs)) in
- let whfun = whd_simpl_stack env sigma in
- (special_red_case env sigma whfun (EConstr.destCase sigma c'), lrest), nocase
+ let c', lrest = whd_nothing_for_iota env sigma (c, largs) in
+ (special_red_case env sigma (EConstr.destCase sigma c'), lrest), nocase
| EliminationProj n when nargs >= n ->
let c = reference_value env sigma ref u in
- let c', lrest = whd_nothing_for_iota env sigma (applist(c,largs)) in
- let whfun = whd_construct_stack env sigma in
- let whfun' = whd_simpl_stack env sigma in
- (reduce_proj env sigma whfun whfun' c', lrest), nocase
+ let c', lrest = whd_nothing_for_iota env sigma (c, largs) in
+ (reduce_proj env sigma c', lrest), nocase
| EliminationFix (min,minfxargs,infos) when nargs >= min ->
let c = reference_value env sigma ref u in
- let d, lrest = whd_nothing_for_iota env sigma (applist(c,largs)) in
- let f = make_elim_fun ([|Some (minfxargs,ref)|],infos) u largs in
- let whfun = whd_construct_stack env sigma in
- (match reduce_fix_use_function env sigma f whfun (destFix sigma d) lrest with
+ let d, lrest = whd_nothing_for_iota env sigma (c, largs) in
+ let f = ([|Some (minfxargs,ref)|],infos), u, largs in
+ (match reduce_fix_use_function env sigma f (destFix sigma d) lrest with
| NotReducible -> raise Redelimination
| Reduced (c,rest) -> (nf_beta env sigma c, rest), nocase)
| EliminationMutualFix (min,refgoal,refinfos) when nargs >= min ->
@@ -729,10 +649,9 @@ let rec red_elim_const env sigma ref u largs =
let c', lrest = whd_betalet_stack env sigma (applist(c,args)) in
descend (destEvalRefU sigma c') lrest in
let (_, midargs as s) = descend (ref,u) largs in
- let d, lrest = whd_nothing_for_iota env sigma (applist s) in
- let f = make_elim_fun refinfos u midargs in
- let whfun = whd_construct_stack env sigma in
- (match reduce_fix_use_function env sigma f whfun (destFix sigma d) lrest with
+ let d, lrest = whd_nothing_for_iota env sigma s in
+ let f = refinfos, u, midargs in
+ (match reduce_fix_use_function env sigma f (destFix sigma d) lrest with
| NotReducible -> raise Redelimination
| Reduced (c,rest) -> (nf_beta env sigma c, rest), nocase)
| NotAnElimination when unfold_nonelim ->
@@ -755,32 +674,30 @@ and reduce_params env sigma stack l =
| _ -> raise Redelimination)
stack l
-
(* reduce to whd normal form or to an applied constant that does not hide
a reducible iota/fix/cofix redex (the "simpl" tactic) *)
and whd_simpl_stack env sigma =
let open ReductionBehaviour in
let rec redrec s =
- let (x, stack) = decompose_app_vect sigma s in
- let stack = Array.to_list stack in
- let s' = (x, stack) in
+ let s' = push_app sigma s in
+ let (x, stack) = s' in
match EConstr.kind sigma x with
| Lambda (na,t,c) ->
(match stack with
| [] -> s'
- | a :: rest -> redrec (beta_applist sigma (x, stack)))
- | LetIn (n,b,t,c) -> redrec (applist (Vars.substl [b] c, stack))
- | App (f,cl) -> redrec (applist(f, (Array.to_list cl)@stack))
- | Cast (c,_,_) -> redrec (applist(c, stack))
+ | a :: rest -> redrec (beta_applist sigma [a] c rest))
+ | LetIn (n,b,t,c) -> redrec (Vars.substl [b] c, stack)
+ | App (f,cl) -> assert false (* see push_app above *)
+ | Cast (c,_,_) -> redrec (c, stack)
| Case (ci,p,iv,c,lf) ->
(try
- redrec (applist(special_red_case env sigma redrec (ci,p,iv,c,lf), stack))
+ redrec (special_red_case env sigma (ci,p,iv,c,lf), stack)
with
Redelimination -> s')
| Fix fix ->
- (try match reduce_fix (whd_construct_stack env) sigma fix stack with
- | Reduced s' -> redrec (applist s')
+ (try match reduce_fix env sigma fix stack with
+ | Reduced s' -> redrec s'
| NotReducible -> s'
with Redelimination -> s')
@@ -800,11 +717,11 @@ and whd_simpl_stack env sigma =
(match reduce_projection env sigma p ~npars
(whd_construct_stack env sigma c) stack
with
- | Reduced s' -> redrec (applist s')
+ | Reduced s' -> redrec s'
| NotReducible -> s')
| _ ->
match reduce_projection env sigma p ~npars (whd_construct_stack env sigma c) stack with
- | Reduced s' -> redrec (applist s')
+ | Reduced s' -> redrec s'
| NotReducible -> s')
else s'
with Redelimination -> s')
@@ -814,7 +731,7 @@ and whd_simpl_stack env sigma =
| Some (ref, u) ->
(try
let sapp, nocase = red_elim_const env sigma ref u stack in
- let hd, _ as s'' = redrec (applist(sapp)) in
+ let hd, _ as s'' = redrec sapp in
let rec is_case x = match EConstr.kind sigma x with
| Lambda (_,_, x) | LetIn (_,_,_, x) | Cast (x, _,_) -> is_case x
| App (hd, _) -> is_case hd
@@ -827,10 +744,102 @@ and whd_simpl_stack env sigma =
in
redrec
+and reduce_fix env sigma fix stack =
+ match fix_recarg fix stack with
+ | None -> NotReducible
+ | Some (recargnum,recarg) ->
+ let (recarg'hd,_ as recarg') = whd_construct_stack env sigma recarg in
+ let stack' = List.assign stack recargnum (applist recarg') in
+ (match EConstr.kind sigma recarg'hd with
+ | Construct _ -> Reduced (contract_fix sigma fix, stack')
+ | _ -> NotReducible)
+
+and reduce_fix_use_function env sigma f fix stack =
+ match fix_recarg fix stack with
+ | None -> NotReducible
+ | Some (recargnum,recarg) ->
+ let (recarg'hd,_ as recarg') =
+ if EConstr.isRel sigma recarg then
+ (* The recarg cannot be a local def, no worry about the right env *)
+ (recarg, [])
+ else
+ whd_construct_stack env sigma recarg in
+ let stack' = List.assign stack recargnum (applist recarg') in
+ (match EConstr.kind sigma recarg'hd with
+ | Construct _ ->
+ let (names, (nbfix, lv, n)), u, largs = f in
+ let lu = List.firstn n largs in
+ let p = List.length lv in
+ let lyi = List.map fst lv in
+ let la =
+ List.map_i (fun q aq ->
+ (* k from the comment is q+1 *)
+ try mkRel (p+1-(List.index Int.equal (n-q) lyi))
+ with Not_found -> Vars.lift p aq)
+ 0 lu
+ in
+ let f i = match names.(i) with
+ | None -> None
+ | Some (minargs,ref) ->
+ let body = applist (mkEvalRef ref u, la) in
+ let g =
+ List.fold_left_i (fun q (* j = n+1-q *) c (ij,tij) ->
+ let subst = List.map (Vars.lift (-q)) (List.firstn (n-ij) la) in
+ let tij' = Vars.substl (List.rev subst) tij in
+ let x = make_annot x Sorts.Relevant in (* TODO relevance *)
+ mkLambda (x,tij',c)) 1 body (List.rev lv)
+ in Some (minargs,g)
+ in
+ Reduced (contract_fix_use_function env sigma f fix,stack')
+ | _ -> NotReducible)
+
+and reduce_proj env sigma c =
+ let rec redrec s =
+ match EConstr.kind sigma s with
+ | Proj (proj, c) ->
+ let c' = try redrec c with Redelimination -> c in
+ let constr, cargs = whd_construct_stack env sigma c' in
+ (match EConstr.kind sigma constr with
+ | Construct _ ->
+ let proj_narg = Projection.npars proj + Projection.arg proj in
+ List.nth cargs proj_narg
+ | _ -> raise Redelimination)
+ | Case (n,p,iv,c,brs) ->
+ let c' = redrec c in
+ let p = (n,p,iv,c',brs) in
+ (try special_red_case env sigma p
+ with Redelimination -> mkCase p)
+ | _ -> raise Redelimination
+ in redrec c
+
+and special_red_case env sigma (ci, p, iv, c, lf) =
+ let rec redrec s =
+ let (constr, cargs) = whd_simpl_stack env sigma s in
+ match match_eval_ref env sigma constr cargs with
+ | Some (ref, u) ->
+ (match reference_opt_value env sigma ref u with
+ | None -> raise Redelimination
+ | Some gvalue ->
+ if reducible_mind_case sigma gvalue then
+ reduce_mind_case_use_function constr env sigma
+ {mP=p; mconstr=gvalue; mcargs=cargs;
+ mci=ci; mlf=lf}
+ else
+ redrec (gvalue, cargs))
+ | None ->
+ if reducible_mind_case sigma constr then
+ reduce_mind_case sigma
+ {mP=p; mconstr=constr; mcargs=cargs;
+ mci=ci; mlf=lf}
+ else
+ raise Redelimination
+ in
+ redrec (push_app sigma (c, []))
+
(* reduce until finding an applied constructor or fail *)
and whd_construct_stack env sigma s =
- let (constr, cargs as s') = whd_simpl_stack env sigma s in
+ let (constr, cargs as s') = whd_simpl_stack env sigma (s, []) in
if reducible_mind_case sigma constr then s'
else match match_eval_ref env sigma constr cargs with
| Some (ref, u) ->
@@ -855,13 +864,13 @@ let try_red_product env sigma c =
| App (f,l) ->
(match EConstr.kind sigma f with
| Fix fix ->
- let stack = Stack.append_app l Stack.empty in
- (match fix_recarg fix stack with
+ (match fix_recarg fix (Array.to_list l) with
| None -> raise Redelimination
| Some (recargnum,recarg) ->
let recarg' = redrec env recarg in
- let stack' = Stack.assign stack recargnum recarg' in
- simpfun (Stack.zip sigma (f,stack')))
+ let l = Array.copy l in
+ let () = Array.set l recargnum recarg' in
+ simpfun (mkApp (f, l)))
| _ -> simpfun (mkApp (redrec env f, l)))
| Cast (c,_,_) -> redrec env c
| Prod (x,a,b) ->
@@ -973,19 +982,19 @@ let whd_simpl_orelse_delta_but_fix env sigma c =
if List.length stack <= npars then
(* Do not show the eta-expanded form *)
s'
- else redrec (applist (c, stack))
- | _ -> redrec (applist(c, stack)))
+ else redrec (c, stack)
+ | _ -> redrec (c, stack))
| None -> s'
in
let simpfun = clos_norm_flags betaiota env sigma in
simpfun (applist (redrec c))
-let hnf_constr = whd_simpl_orelse_delta_but_fix
+let hnf_constr env sigma c = whd_simpl_orelse_delta_but_fix env sigma (c, [])
(* The "simpl" reduction tactic *)
let whd_simpl env sigma c =
- applist (whd_simpl_stack env sigma c)
+ applist (whd_simpl_stack env sigma (c, []))
let simpl env sigma c = strong whd_simpl env sigma c
@@ -1267,11 +1276,10 @@ let one_step_reduce env sigma c =
| Cast (c,_,_) -> redrec (c,stack)
| Case (ci,p,iv,c,lf) ->
(try
- (special_red_case env sigma (whd_simpl_stack env sigma)
- (ci,p,iv,c,lf), stack)
+ (special_red_case env sigma (ci,p,iv,c,lf), stack)
with Redelimination -> raise NotStepReducible)
| Fix fix ->
- (try match reduce_fix (whd_construct_stack env) sigma fix stack with
+ (try match reduce_fix env sigma fix stack with
| Reduced s' -> s'
| NotReducible -> raise NotStepReducible
with Redelimination -> raise NotStepReducible)