aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/quote
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-11-25 18:34:53 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2017-02-14 17:30:41 +0100
commit02dd160233adc784eac732d97a88356d1f0eaf9b (patch)
treed2baacdc2a4ae06e4607bfe09b48ba2c23a78a0f /plugins/quote
parenta5499688bd76def8de3d8e1089a49c7a08430903 (diff)
Removing various compatibility layers of tactics.
Diffstat (limited to 'plugins/quote')
-rw-r--r--plugins/quote/quote.ml6
1 files changed, 2 insertions, 4 deletions
diff --git a/plugins/quote/quote.ml b/plugins/quote/quote.ml
index 87276f5df..edf34607b 100644
--- a/plugins/quote/quote.ml
+++ b/plugins/quote/quote.ml
@@ -459,8 +459,7 @@ let quote f lid =
let env = Proofview.Goal.env gl in
let sigma = Tacmach.New.project gl in
let f = Tacmach.New.pf_global f gl in
- let f = EConstr.of_constr f in
- let cl = List.map (fun id -> Tacmach.New.pf_global id gl) lid in
+ let cl = List.map (fun id -> EConstr.to_constr sigma (Tacmach.New.pf_global id gl)) lid in
let ivs = compute_ivs f cl gl in
let concl = Proofview.Goal.concl gl in
let quoted_terms = quote_terms env sigma ivs [concl] in
@@ -478,8 +477,7 @@ let gen_quote cont c f lid =
let env = Proofview.Goal.env gl in
let sigma = Tacmach.New.project gl in
let f = Tacmach.New.pf_global f gl in
- let f = EConstr.of_constr f in
- let cl = List.map (fun id -> Tacmach.New.pf_global id gl) lid in
+ let cl = List.map (fun id -> EConstr.to_constr sigma (Tacmach.New.pf_global id gl)) lid in
let ivs = compute_ivs f cl gl in
let quoted_terms = quote_terms env sigma ivs [c] in
let (p, vm) = match quoted_terms with