diff options
author | aspiwack <aspiwack@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2012-04-18 14:47:40 +0000 |
---|---|---|
committer | aspiwack <aspiwack@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2012-04-18 14:47:40 +0000 |
commit | 676f63e7b5e0803cf7bee756369323b4ea42052b (patch) | |
tree | 442c013092b2d7fc2e4730cfaa7bfb96e1b05687 /tactics | |
parent | e984ac1984bb1e2d102b6c3c93ddcbdd5f689b23 (diff) |
Adds the openconstr entry for tactic notations.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@15206 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tactics')
-rw-r--r-- | tactics/tacinterp.ml | 9 |
1 files changed, 9 insertions, 0 deletions
diff --git a/tactics/tacinterp.ml b/tactics/tacinterp.ml index b03923bcc..5b2a932e5 100644 --- a/tactics/tacinterp.ml +++ b/tactics/tacinterp.ml @@ -1727,6 +1727,9 @@ let apply_one_mhyp_context ist env gl lmatch (hypname,patv,pat) lhyps = (* misc *) let mk_constr_value ist gl c = VConstr ([],pf_interp_constr ist gl c) +let mk_open_constr_value ist gl c = + let (sigma,c_interp) = pf_apply (interp_open_constr None ist) gl c in + sigma,VConstr ([],c_interp) let mk_hyp_value ist gl c = VConstr ([],mkVar (interp_hyp ist gl c)) let mk_int_or_var_value ist c = VInteger (interp_int_or_var ist c) @@ -2391,6 +2394,7 @@ and interp_atomic ist gl tac = let args = List.map (interp_genarg ist gl) l in abstract_extended_tactic opn args (tac args) | TacAlias (loc,s,l,(_,body)) -> fun gl -> + let evdref = ref gl.sigma in let rec f x = match genarg_tag x with | IntArgType -> VInteger (out_gen globwit_int x) @@ -2413,6 +2417,10 @@ and interp_atomic ist gl tac = VConstr ([],mkSort (interp_sort (out_gen globwit_sort x))) | ConstrArgType -> mk_constr_value ist gl (out_gen globwit_constr x) + | OpenConstrArgType false -> + let (sigma,v) = mk_open_constr_value ist gl (snd (out_gen globwit_open_constr x)) in + evdref := sigma; + v | ConstrMayEvalArgType -> VConstr ([],interp_constr_may_eval ist gl (out_gen globwit_constr_may_eval x)) @@ -2471,6 +2479,7 @@ and interp_atomic ist gl tac = in let lfun = (List.map (fun (x,c) -> (x,f c)) l)@ist.lfun in let trace = push_trace (loc,LtacNotationCall s) ist.trace in + let gl = { gl with sigma = !evdref } in interp_tactic { ist with lfun=lfun; trace=trace } body gl let make_empty_glob_sign () = |