aboutsummaryrefslogtreecommitdiff
path: root/kernel/reduction.ml
diff options
context:
space:
mode:
authorfilliatr2000-11-22 15:09:17 +0000
committerfilliatr2000-11-22 15:09:17 +0000
commitdcfeca5f828bc2648b567616e3dfabd03e13d9ab (patch)
treee6ff8cddaa26116cd023bc30e790aa6aa2da0f61 /kernel/reduction.ml
parent24cb368c8cda29daa0c34a807e49146c4885226a (diff)
deplacement poly_args; iterateurs sur les segments
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@917 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'kernel/reduction.ml')
-rw-r--r--kernel/reduction.ml34
1 files changed, 0 insertions, 34 deletions
diff --git a/kernel/reduction.ml b/kernel/reduction.ml
index dd2adf2f5f..d496a9e49a 100644
--- a/kernel/reduction.ml
+++ b/kernel/reduction.ml
@@ -1104,40 +1104,6 @@ let is_info_type env sigma t =
(s <> Prop Null &&
try info_arity env sigma t.utj_val with IsType -> true)
-(* calcul des arguments implicites *)
-
-(* la seconde liste est ordonne'e *)
-
-let ord_add x l =
- let rec aux l = match l with
- | [] -> [x]
- | y::l' -> if y > x then x::l else if x = y then l else y::(aux l')
- in
- aux l
-
-let add_free_rels_until bound m acc =
- let rec frec depth acc c = match kind_of_term c with
- | IsRel n when (n < bound+depth) & (n >= depth) ->
- Intset.add (bound+depth-n) acc
- | _ -> fold_constr_with_binders succ frec depth acc c
- in
- frec 1 acc m
-
-(* calcule la liste des arguments implicites *)
-
-let poly_args env sigma t =
- let rec aux env n t =
- match kind_of_term (whd_betadeltaiota env sigma t) with
- | IsProd (x,a,b) ->
- add_free_rels_until n a
- (aux (push_rel_assum (x,a) env) (n+1) b)
- | _ -> Intset.empty
- in
- match kind_of_term (whd_betadeltaiota env sigma t) with
- | IsProd (x,a,b) ->
- Intset.elements (aux (push_rel_assum (x,a) env) 1 b)
- | _ -> []
-
(* Expanding existential variables (pretyping.ml) *)
(* 1- whd_ise fails if an existential is undefined *)