aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-03-29 14:06:47 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-03-29 14:06:47 +0000
commit67787e6daeb7bf2fe59d5546969197ca9f87c2dc (patch)
treecb5d2bb991afcfcb53d879aa37d2a2187c90ca9c /pretyping
parent5193d92186e14794a346392af4d80fc264d8fff7 (diff)
Mise en place de 'Implicit Variable' (variante du 'Reserve' de mizar)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3806 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'pretyping')
-rw-r--r--pretyping/detyping.ml6
-rw-r--r--pretyping/rawterm.ml4
-rw-r--r--pretyping/rawterm.mli2
3 files changed, 6 insertions, 6 deletions
diff --git a/pretyping/detyping.ml b/pretyping/detyping.ml
index f676717d7..c2578cdd7 100644
--- a/pretyping/detyping.ml
+++ b/pretyping/detyping.ml
@@ -272,18 +272,18 @@ let rec detype tenv avoid env t =
let rec remove_type avoid args c =
match c,args with
| RLambda (loc,na,t,c), _::args ->
- let h = RHole (loc,AbstractionType na) in
+ let h = RHole (loc,BinderType na) in
RLambda (loc,na,h,remove_type avoid args c)
| RLetIn (loc,na,b,c), _::args ->
RLetIn (loc,na,b,remove_type avoid args c)
| c, (na,None,t)::args ->
let id = next_name_away_with_default "x" na avoid in
- let h = RHole (dummy_loc,AbstractionType na) in
+ let h = RHole (dummy_loc,BinderType na) in
let c = remove_type (id::avoid) args
(RApp (dummy_loc,c,[RVar (dummy_loc,id)])) in
RLambda (dummy_loc,Name id,h,c)
| c, (na,Some b,t)::args ->
- let h = RHole (dummy_loc,AbstractionType na) in
+ let h = RHole (dummy_loc,BinderType na) in
let avoid = name_fold (fun x l -> x::l) na avoid in
RLetIn (dummy_loc,na,h,remove_type avoid args c)
| c, [] -> c in
diff --git a/pretyping/rawterm.ml b/pretyping/rawterm.ml
index 77afa8041..0075be7d8 100644
--- a/pretyping/rawterm.ml
+++ b/pretyping/rawterm.ml
@@ -50,7 +50,7 @@ type 'a with_bindings = 'a * 'a substitution
type hole_kind =
| ImplicitArg of global_reference * int
- | AbstractionType of name
+ | BinderType of name
| QuestionMark
| CasesType
| InternalHole
@@ -235,7 +235,7 @@ let rec subst_raw subst raw =
let ref' = subst_global subst ref in
if ref' == ref then raw else
RHole (loc,ImplicitArg (ref',i))
- | RHole (loc, (AbstractionType _ | QuestionMark | CasesType |
+ | RHole (loc, (BinderType _ | QuestionMark | CasesType |
InternalHole | TomatchTypeParameter _)) -> raw
| RCast (loc,r1,r2) ->
diff --git a/pretyping/rawterm.mli b/pretyping/rawterm.mli
index b5e408bb5..7ac8a15b7 100644
--- a/pretyping/rawterm.mli
+++ b/pretyping/rawterm.mli
@@ -48,7 +48,7 @@ type 'a with_bindings = 'a * 'a substitution
type hole_kind =
| ImplicitArg of global_reference * int
- | AbstractionType of name
+ | BinderType of name
| QuestionMark
| CasesType
| InternalHole