aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-10-26 22:33:45 +0100
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-10-27 09:57:11 +0100
commita9adcb3941900c416f106ddac6fd646603b335b8 (patch)
tree0c86b8c13cfd06179b96b72aeb2896cee3bdd272
parent65c8d91cd4c11b8de44f0b23cd44a3303cd54d4e (diff)
Dead code
-rw-r--r--parsing/g_tactic.ml47
-rw-r--r--pretyping/unification.ml2
2 files changed, 1 insertions, 8 deletions
diff --git a/parsing/g_tactic.ml4 b/parsing/g_tactic.ml4
index 25dd0db45..fb09a3108 100644
--- a/parsing/g_tactic.ml4
+++ b/parsing/g_tactic.ml4
@@ -619,13 +619,6 @@ GEXTEND Gram
l = LIST0 [","; c = pattern_occ; na = as_name -> (c,na)] ->
TacAtom (!@loc, TacGeneralize (((nl,c),na)::l))
| IDENT "generalize"; IDENT "dependent"; c = constr -> TacAtom (!@loc, TacGeneralizeDep c)
-(* Towards a "generalize in" which generalize in place: problem: this is somehow inconsistent with "generalize at" (from 8.2) which is not in place.
- | IDENT "generalize"; c = constr; "in"; cl = in_clause;
- na = as_name;
- l = LIST0 [","; c = constr; "in"; cl = in_clause; na = as_name ->
- ((cl,c),na)] ->
- TacGeneralize (true,((cl,c),na)::l)
-*)
(* Derived basic tactics *)
| IDENT "induction"; ic = induction_clause_list ->
diff --git a/pretyping/unification.ml b/pretyping/unification.ml
index 1a1d03cc8..07940bf57 100644
--- a/pretyping/unification.ml
+++ b/pretyping/unification.ml
@@ -1480,7 +1480,7 @@ let make_abstraction_core name (test,out) env sigma c ty occs check_occs concl =
++ str ".")
else
(push_named_context_val d sign,depdecls)
- | (AtOccs (AllOccurrences, InHyp) | LikeFirst) as occ ->
+ | (AtOccs (AllOccurrences, InHyp) | LikeFirst) ->
let newdecl = replace_term_occ_decl_modulo LikeFirst test mkvarid d in
if Context.eq_named_declaration d newdecl
&& not (indirectly_dependent c d depdecls)