aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-01-24 17:13:29 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-01-24 17:13:29 +0000
commitfb20fe8c71c7bbd1f8100c8d60ebb2f52afa8b16 (patch)
treea58564d6800c8c1a85e4511cb0c2bdbd7c0e898a /pretyping
parent0b6a729e05b0b120f8d0a34b135bb0cf7e5bab82 (diff)
code mort
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2429 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'pretyping')
-rw-r--r--pretyping/indrec.ml45
1 files changed, 0 insertions, 45 deletions
diff --git a/pretyping/indrec.ml b/pretyping/indrec.ml
index b60c3a3b2..68739e40e 100644
--- a/pretyping/indrec.ml
+++ b/pretyping/indrec.ml
@@ -169,51 +169,6 @@ let type_rec_branch dep env sigma (vargs,depPvect,decP) tyi cs recargs =
let co = applist (mkConstruct cs.cs_cstr,params@realargs) in
mkApp (c, [|co|])
else c
-(*
- let c', largs = whd_stack c in
- match kind_of_term c' with
- | Prod (n,t,c_0) ->
- let (optionpos,rest) =
- match recargs with
- | [] -> None,[]
- | Param _ :: rest -> (None,rest)
- | Norec :: rest -> (None,rest)
- | Imbr _ :: rest ->
- warning "Ignoring recursive call"; (None,rest)
- | Mrec j :: rest -> (depPvect.(j),rest)
- in
- (match optionpos with
- | None ->
- make_prod env
- (n,t,
- process_constr (push_rel (n,None,t) env) (i+1) c_0 rest
- (mkApp (lift 1 co, [|mkRel 1|])))
- | Some(dep',p) ->
- let nP = lift (i+1+decP) p in
- let t_0 = process_pos env dep' nP (lift 1 t) in
- make_prod_dep (dep or dep') env
- (n,t,
- mkArrow t_0
- (process_constr
- (push_rel (n,None,t)
- (push_rel (Anonymous,None,t_0) env))
- (i+2) (lift 1 c_0) rest
- (mkApp (lift 2 co, [|mkRel 2|])))))
- | LetIn (n,b,t,c_0) ->
- mkLetIn (n,b,t,
- process_constr
- (push_rel (n,Some b,t) env)
- (i+1) c_0 recargs (lift 1 co))
-
- | Ind ((_,tyi),_) ->
- let nP = match depPvect.(tyi) with
- | Some(_,p) -> lift (i+decP) p
- | _ -> assert false in
- let (_,realargs) = list_chop nparams largs in
- let base = applist (nP,realargs) in
- if dep then mkApp (base, [|co|]) else base
- | _ -> assert false
-*)
in
let nhyps = List.length cs.cs_args in
let nP = match depPvect.(tyi) with