aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/goal.ml
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-01-08 09:06:58 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-01-10 17:46:36 +0100
commit6058cdf5e70822e4501c61dfd969e4746c01145b (patch)
tree08a86366100937b2f91742807c3ad76ec0848048 /proofs/goal.ml
parenta6ca35c30199f3ccf0ebb7d9b200190e345c4d50 (diff)
Exporting the full pretyper options in Goal.constr_of_raw.
Diffstat (limited to 'proofs/goal.ml')
-rw-r--r--proofs/goal.ml15
1 files changed, 4 insertions, 11 deletions
diff --git a/proofs/goal.ml b/proofs/goal.ml
index 43d7b3579..c660f403f 100644
--- a/proofs/goal.ml
+++ b/proofs/goal.ml
@@ -232,27 +232,20 @@ module Refinable = struct
many things to go wrong. *)
handle := fusion delta_list !handle
- (* [constr_of_raw] is a pretyping function. The [check_type] argument
- asks whether the term should have the same type as the conclusion.
- [resolve_classes] is a flag on pretyping functions which, if set to true,
- calls the typeclass resolver.
+ (* [constr_of_raw h tycon flags] is a pretyping function.
+ The [tycon] argument allows to put a type constraint on the returned term.
+ The [flags] argument is passed to the pretyper.
The principal argument is a [glob_constr] which is then pretyped in the
context of a term, the remaining evars are registered to the handle.
It is the main component of the toplevel refine tactic.*)
(* spiwack: it is not entirely satisfactory to have this function here. Plus it is
a bit hackish. However it does not seem possible to move it out until
pretyping is defined as some proof procedure. *)
- let constr_of_raw handle check_type resolve_classes lvar rawc = (); fun env rdefs gl info ->
+ let constr_of_raw handle tycon flags lvar rawc = (); fun env rdefs gl info ->
(* We need to keep trace of what [rdefs] was originally*)
let init_defs = !rdefs in
- (* if [check_type] is true, then creates a type constraint for the
- proof-to-be *)
- let tycon = if check_type then Pretyping.OfType (Evd.evar_concl info) else Pretyping.WithoutTypeConstraint in
(* call to [understand_tcc_evars] returns a constr with undefined evars
these evars will be our new goals *)
- let flags =
- if resolve_classes then Pretyping.all_no_fail_flags
- else Pretyping.no_classes_no_fail_inference_flags in
let (sigma, open_constr) =
Pretyping.understand_ltac flags !rdefs env lvar tycon rawc
in