aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-11-21 21:33:14 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2017-02-14 17:30:34 +0100
commita327ae04966aa1c7786ae32157516e934068ea89 (patch)
treea44bc1804aeb7beb90f4eb45d272c439616af7d3 /proofs
parent0cdb7e42f64674e246d4e24e3c725e23ceeec6bd (diff)
Quote API using EConstr.
Diffstat (limited to 'proofs')
-rw-r--r--proofs/tacmach.ml5
-rw-r--r--proofs/tacmach.mli4
2 files changed, 7 insertions, 2 deletions
diff --git a/proofs/tacmach.ml b/proofs/tacmach.ml
index 7ecf0a9e8..d9caadd54 100644
--- a/proofs/tacmach.ml
+++ b/proofs/tacmach.ml
@@ -41,6 +41,11 @@ let project = Refiner.project
let pf_env = Refiner.pf_env
let pf_hyps = Refiner.pf_hyps
+let test_conversion cb env sigma c1 c2 =
+ let c1 = EConstr.Unsafe.to_constr c1 in
+ let c2 = EConstr.Unsafe.to_constr c2 in
+ test_conversion cb env sigma c1 c2
+
let pf_concl gls = EConstr.Unsafe.to_constr (Goal.V82.concl (project gls) (sig_it gls))
let pf_hyps_types gls =
let sign = Environ.named_context (pf_env gls) in
diff --git a/proofs/tacmach.mli b/proofs/tacmach.mli
index 21511b6f9..06b3e3981 100644
--- a/proofs/tacmach.mli
+++ b/proofs/tacmach.mli
@@ -74,8 +74,8 @@ val pf_unfoldn : (occurrences * evaluable_global_reference) list
-> goal sigma -> EConstr.constr -> EConstr.constr
val pf_const_value : goal sigma -> pconstant -> constr
-val pf_conv_x : goal sigma -> constr -> constr -> bool
-val pf_conv_x_leq : goal sigma -> constr -> constr -> bool
+val pf_conv_x : goal sigma -> EConstr.constr -> EConstr.constr -> bool
+val pf_conv_x_leq : goal sigma -> EConstr.constr -> EConstr.constr -> bool
val pf_matches : goal sigma -> constr_pattern -> EConstr.constr -> patvar_map
val pf_is_matching : goal sigma -> constr_pattern -> EConstr.constr -> bool