aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2005-02-18 22:08:16 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2005-02-18 22:08:16 +0000
commit4bc680136b9310f7ab630e41b47314b9efdbe9d2 (patch)
tree7db95e8696f94491eca80be4e591a168909c74ba /tactics
parentbd8f528f2f031751d35fd27f85dba7cdc8cf6df6 (diff)
Moving subst_inductive from tacinterp to inductiveops for better for reuse in recordops
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@6741 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tactics')
-rw-r--r--tactics/tacinterp.ml6
1 files changed, 2 insertions, 4 deletions
diff --git a/tactics/tacinterp.ml b/tactics/tacinterp.ml
index 52ed344a5..87906d01c 100644
--- a/tactics/tacinterp.ml
+++ b/tactics/tacinterp.ml
@@ -1815,7 +1815,7 @@ and interp_atomic ist gl = function
| HypArgType ->
VConstr (mkVar (interp_var ist gl (out_gen globwit_var x)))
| RefArgType ->
- VConstr (constr_of_reference
+ VConstr (constr_of_global
(pf_interp_reference ist gl (out_gen globwit_ref x)))
| SortArgType ->
VConstr (mkSort (Pretyping.interp_sort (out_gen globwit_sort x)))
@@ -1864,8 +1864,6 @@ let subst_quantified_hypothesis _ x = x
let subst_declared_or_quantified_hypothesis _ x = x
-let subst_inductive subst (kn,i) = (subst_kn subst kn,i)
-
let subst_rawconstr subst (c,e) =
assert (e=None); (* e<>None only for toplevel tactics *)
(Detyping.subst_raw subst c,None)
@@ -1905,7 +1903,7 @@ let subst_reference subst =
let subst_global_reference subst =
let subst_global ref =
let ref',t' = subst_global subst ref in
- if not (eq_constr (constr_of_reference ref') t') then
+ if not (eq_constr (constr_of_global ref') t') then
ppnl (str "Warning: the reference " ++ pr_global ref ++ str " is not " ++
str " expanded to \"" ++ prterm t' ++ str "\", but to " ++
pr_global ref') ;