aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping/cases.ml
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-11-26 15:30:02 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2017-02-14 17:30:43 +0100
commit78a8d59b39dfcb07b94721fdcfd9241d404905d2 (patch)
tree96cc7802206b80a19cc4760855357636892f9b9e /pretyping/cases.ml
parentc8c8ccdaaffefdbd3d78c844552a08bcb7b4f915 (diff)
Introducing contexts parameterized by the inner term type.
This allows the decoupling of the notions of context containing kernel terms and context containing tactic-level terms.
Diffstat (limited to 'pretyping/cases.ml')
-rw-r--r--pretyping/cases.ml2
1 files changed, 1 insertions, 1 deletions
diff --git a/pretyping/cases.ml b/pretyping/cases.ml
index 0e4c6619b..3b5662a24 100644
--- a/pretyping/cases.ml
+++ b/pretyping/cases.ml
@@ -943,7 +943,7 @@ let abstract_predicate env sigma indf cur realargs (names,na) tms ccl =
let tms = List.fold_right2 (fun par arg tomatch ->
match EConstr.kind sigma par with
| Rel i -> relocate_index_tomatch sigma (i+n) (destRel sigma arg) tomatch
- | _ -> tomatch) (realargs@[cur]) (List.map EConstr.of_constr (Context.Rel.to_extended_list 0 sign))
+ | _ -> tomatch) (realargs@[cur]) (Context.Rel.to_extended_list EConstr.mkRel 0 sign)
(lift_tomatch_stack n tms) in
(* Pred is already dependent in the current term to match (if *)
(* (na<>Anonymous) and its realargs; we just need to adjust it to *)