aboutsummaryrefslogtreecommitdiff
path: root/interp
diff options
context:
space:
mode:
authorHugo Herbelin2014-08-15 17:43:35 +0200
committerHugo Herbelin2014-08-18 18:56:39 +0200
commit5dcafa956e49eefc451dd021a0fe8ad2e2338088 (patch)
treec851c0f1cb32815bae652309c39f6d4a681fd2cc /interp
parent72498d6d68ac12ba4db0db7d54f0ac6fdaaf0c61 (diff)
Lazy interpretation of patterns so that expressions such as "intros H H'/H"
can be given with second H bound by the first one. Not very satisfied by passing closure to tactics.ml, but otherwise tactics would have to be aware of glob_constr.
Diffstat (limited to 'interp')
-rw-r--r--interp/constrarg.ml2
-rw-r--r--interp/constrarg.mli3
2 files changed, 2 insertions, 3 deletions
diff --git a/interp/constrarg.ml b/interp/constrarg.ml
index 9c1382ba14..67282e5dda 100644
--- a/interp/constrarg.ml
+++ b/interp/constrarg.ml
@@ -24,7 +24,7 @@ let unsafe_of_type (t : argument_type) : ('a, 'b, 'c) Genarg.genarg_type =
let wit_int_or_var = unsafe_of_type IntOrVarArgType
-let wit_intro_pattern : (Constrexpr.constr_expr intro_pattern_expr located, glob_constr_and_expr intro_pattern_expr located, constr intro_pattern_expr located) genarg_type =
+let wit_intro_pattern : (Constrexpr.constr_expr intro_pattern_expr located, glob_constr_and_expr intro_pattern_expr located, intro_pattern) genarg_type =
Genarg.make0 None "intropattern"
let wit_tactic : (raw_tactic_expr, glob_tactic_expr, glob_tactic_expr) genarg_type =
diff --git a/interp/constrarg.mli b/interp/constrarg.mli
index b6ff3c850a..ab3d7eafd3 100644
--- a/interp/constrarg.mli
+++ b/interp/constrarg.mli
@@ -28,8 +28,7 @@ val loc_of_or_by_notation : ('a -> Loc.t) -> 'a or_by_notation -> Loc.t
val wit_int_or_var : int or_var uniform_genarg_type
-val wit_intro_pattern : (constr_expr intro_pattern_expr located, glob_constr_and_expr intro_pattern_expr located, constr intro_pattern_expr located) genarg_type
-
+val wit_intro_pattern : (constr_expr intro_pattern_expr located, glob_constr_and_expr intro_pattern_expr located, intro_pattern) genarg_type
val wit_ident : Id.t uniform_genarg_type