aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping/detyping.ml
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-04-26 14:06:42 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-04-26 14:06:42 +0000
commit5db206a826ed54bb9aa1c32f80a729ac326b58f9 (patch)
tree7f145499d593ea30b150dfa8fe3f324e6e7e5dba /pretyping/detyping.ml
parentd488b3bff54732a8e05f9bd48c66695b461ef3af (diff)
N'importe quel rawconstr maintenant dans le contexte d'une référence
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@369 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'pretyping/detyping.ml')
-rw-r--r--pretyping/detyping.ml14
1 files changed, 8 insertions, 6 deletions
diff --git a/pretyping/detyping.ml b/pretyping/detyping.ml
index 32d08d1cd..2dd49e4b7 100644
--- a/pretyping/detyping.ml
+++ b/pretyping/detyping.ml
@@ -254,12 +254,14 @@ let computable p k =
in
striprec (k,p)
+(*
let ids_of_var cl =
List.map
(function
| RRef (_,RVar id) -> id
| _-> anomaly "ids_of_var")
(Array.to_list cl)
+*)
let lookup_name_as_renamed env t s =
let rec lookup avoid env n = function
@@ -313,17 +315,17 @@ let rec detype avoid env t =
| IsAppL (f,args) ->
RApp (dummy_loc,detype avoid env f,List.map (detype avoid env) args)
| IsConst (sp,cl) ->
- RRef(dummy_loc,RConst(sp,ids_of_var (Array.map (detype avoid env) cl)))
+ RRef(dummy_loc,RConst(sp,Array.map (detype avoid env) cl))
| IsEvar (ev,cl) ->
- RRef(dummy_loc,REVar(ev,ids_of_var (Array.map (detype avoid env) cl)))
+ RRef(dummy_loc,REVar(ev,Array.map (detype avoid env) cl))
| IsAbst (sp,cl) ->
anomaly "bdize: Abst should no longer occur in constr"
| IsMutInd (ind_sp,cl) ->
- let ids = ids_of_var (Array.map (detype avoid env) cl) in
- RRef (dummy_loc,RInd (ind_sp,ids))
+ let ctxt = Array.map (detype avoid env) cl in
+ RRef (dummy_loc,RInd (ind_sp,ctxt))
| IsMutConstruct (cstr_sp,cl) ->
- let ids = ids_of_var (Array.map (detype avoid env) cl) in
- RRef (dummy_loc,RConstruct (cstr_sp,ids))
+ let ctxt = Array.map (detype avoid env) cl in
+ RRef (dummy_loc,RConstruct (cstr_sp,ctxt))
| IsMutCase (annot,p,c,bl) ->
let synth_type = synthetize_type () in
let tomatch = detype avoid env c in