aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-11-27 10:33:24 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-11-27 10:33:24 +0000
commite39d865bbd2013ef1ef811aafbf0ddcd7a691f6e (patch)
tree0c3019523c5064ca6fb5da2f0cde1225a7f9341f /pretyping
parente4e440a958ce9c49a39f01a3aaeb7603f77cd0a2 (diff)
Utilisation de Let In pour les constantes locales, prise en compte des Let In dans le discharge, l'unification de evarconv et l'unification de clenv
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@979 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'pretyping')
-rw-r--r--pretyping/evarconv.ml199
1 files changed, 105 insertions, 94 deletions
diff --git a/pretyping/evarconv.ml b/pretyping/evarconv.ml
index 3316e2381..c90dcddb1 100644
--- a/pretyping/evarconv.ml
+++ b/pretyping/evarconv.ml
@@ -12,6 +12,26 @@ open Classops
open Recordops
open Evarutil
+
+type flexible_term = FConst of constant | FRel of int | FVar of identifier
+type flex_kind_of_term =
+ | Rigid of constr
+ | MaybeFlexible of flexible_term
+ | Flexible of existential
+
+let flex_kind_of_term c =
+ match kind_of_term c with
+ | IsConst c -> MaybeFlexible (FConst c)
+ | IsRel n -> MaybeFlexible (FRel n)
+ | IsVar id -> MaybeFlexible (FVar id)
+ | IsEvar ev -> Flexible ev
+ | _ -> Rigid c
+
+let eval_flexible_term env = function
+ | FConst c -> constant_opt_value env c
+ | FRel n -> option_app (lift n) (lookup_rel_value n env)
+ | FVar id -> lookup_named_value id env
+
let evar_apprec env isevars stack c =
let rec aux s =
let (t,stack as s') = Reduction.apprec env !isevars s in
@@ -53,8 +73,8 @@ let rec evar_conv_x env isevars pbty term1 term2 =
and evar_eqappr_x env isevars pbty (term1,l1 as appr1) (term2,l2 as appr2) =
(* Evar must be undefined since we have whd_ised *)
- match (kind_of_term term1, kind_of_term term2) with
- | IsEvar (sp1,al1 as ev1), IsEvar (sp2,al2 as ev2) ->
+ match (flex_kind_of_term term1, flex_kind_of_term term2) with
+ | Flexible (sp1,al1 as ev1), Flexible (sp2,al2 as ev2) ->
let f1 () =
if List.length l1 > List.length l2 then
let (deb1,rest1) = list_chop (List.length l1-List.length l2) l1 in
@@ -73,7 +93,7 @@ and evar_eqappr_x env isevars pbty (term1,l1 as appr1) (term2,l2 as appr2) =
in
ise_try isevars [f1; f2]
- | IsEvar ev1, IsConst cst2 ->
+ | Flexible ev1, MaybeFlexible flex2 ->
let f1 () =
(List.length l1 <= List.length l2) &
let (deb2,rest2) = list_chop (List.length l2-List.length l1) l2 in
@@ -81,7 +101,7 @@ and evar_eqappr_x env isevars pbty (term1,l1 as appr1) (term2,l2 as appr2) =
(pbty,ev1,applist(term2,deb2))
& list_for_all2eq (evar_conv_x env isevars CONV) l1 rest2
and f4 () =
- match constant_opt_value env cst2 with
+ match eval_flexible_term env flex2 with
| Some v2 ->
evar_eqappr_x env isevars pbty
appr1 (evar_apprec env isevars l2 v2)
@@ -89,7 +109,7 @@ and evar_eqappr_x env isevars pbty (term1,l1 as appr1) (term2,l2 as appr2) =
in
ise_try isevars [f1; f4]
- | IsConst cst1, IsEvar ev2 ->
+ | MaybeFlexible flex1, Flexible ev2 ->
let f1 () =
(List.length l2 <= List.length l1) &
let (deb1,rest1) = list_chop (List.length l1-List.length l2) l1 in
@@ -97,7 +117,7 @@ and evar_eqappr_x env isevars pbty (term1,l1 as appr1) (term2,l2 as appr2) =
(pbty,ev2,applist(term1,deb1))
& list_for_all2eq (evar_conv_x env isevars CONV) rest1 l2
and f4 () =
- match constant_opt_value env cst1 with
+ match eval_flexible_term env flex1 with
| Some v1 ->
evar_eqappr_x env isevars pbty
(evar_apprec env isevars l1 v1) appr2
@@ -105,10 +125,9 @@ and evar_eqappr_x env isevars pbty (term1,l1 as appr1) (term2,l2 as appr2) =
in
ise_try isevars [f1; f4]
- | IsConst (sp1,al1 as cst1), IsConst (sp2,al2 as cst2) ->
+ | MaybeFlexible flex1, MaybeFlexible flex2 ->
let f2 () =
- (sp1 = sp2)
- & (array_for_all2 (evar_conv_x env isevars CONV) al1 al2)
+ (flex1 = flex2)
& (list_for_all2eq (evar_conv_x env isevars CONV) l1 l2)
and f3 () =
(try conv_record env isevars
@@ -116,12 +135,12 @@ and evar_eqappr_x env isevars pbty (term1,l1 as appr1) (term2,l2 as appr2) =
with Not_found -> check_conv_record appr2 appr1)
with _ -> false)
and f4 () =
- match constant_opt_value env cst2 with
+ match eval_flexible_term env flex2 with
| Some v2 ->
evar_eqappr_x env isevars pbty
appr1 (evar_apprec env isevars l2 v2)
| None ->
- match constant_opt_value env cst1 with
+ match eval_flexible_term env flex1 with
| Some v1 ->
evar_eqappr_x env isevars pbty
(evar_apprec env isevars l1 v1) appr2
@@ -129,26 +148,26 @@ and evar_eqappr_x env isevars pbty (term1,l1 as appr1) (term2,l2 as appr2) =
in
ise_try isevars [f2; f3; f4]
- | IsEvar ev1, _ ->
+ | Flexible ev1, Rigid _ ->
(List.length l1 <= List.length l2) &
let (deb2,rest2) = list_chop (List.length l2-List.length l1) l2 in
solve_simple_eqn evar_conv_x env isevars
(pbty,ev1,applist(term2,deb2))
& list_for_all2eq (evar_conv_x env isevars CONV) l1 rest2
- | _, IsEvar ev2 ->
+ | Rigid _, Flexible ev2 ->
(List.length l2 <= List.length l1) &
let (deb1,rest1) = list_chop (List.length l1-List.length l2) l1 in
solve_simple_eqn evar_conv_x env isevars
(pbty,ev2,applist(term1,deb1))
& list_for_all2eq (evar_conv_x env isevars CONV) rest1 l2
- | IsConst cst1, _ ->
+ | MaybeFlexible flex1, Rigid _ ->
let f3 () =
(try conv_record env isevars (check_conv_record appr1 appr2)
with _ -> false)
and f4 () =
- match constant_opt_value env cst1 with
+ match eval_flexible_term env flex1 with
| Some v1 ->
evar_eqappr_x env isevars pbty
(evar_apprec env isevars l1 v1) appr2
@@ -156,12 +175,12 @@ and evar_eqappr_x env isevars pbty (term1,l1 as appr1) (term2,l2 as appr2) =
in
ise_try isevars [f3; f4]
- | _ , IsConst cst2 ->
+ | Rigid _ , MaybeFlexible flex2 ->
let f3 () =
(try (conv_record env isevars (check_conv_record appr2 appr1))
with _ -> false)
and f4 () =
- match constant_opt_value env cst2 with
+ match eval_flexible_term env flex2 with
| Some v2 ->
evar_eqappr_x env isevars pbty
appr1 (evar_apprec env isevars l2 v2)
@@ -169,89 +188,81 @@ and evar_eqappr_x env isevars pbty (term1,l1 as appr1) (term2,l2 as appr2) =
in
ise_try isevars [f3; f4]
- | IsRel n, IsRel m ->
- n=m
- & (List.length(l1) = List.length(l2))
- & (List.for_all2 (evar_conv_x env isevars CONV) l1 l2)
-
- | IsCast (c1,_), _ -> evar_eqappr_x env isevars pbty (c1,l1) appr2
-
- | _, IsCast (c2,_) -> evar_eqappr_x env isevars pbty appr1 (c2,l2)
-
- | IsVar id1, IsVar id2 ->
- (id1=id2 & (List.length l1 = List.length l2)
- & (List.for_all2 (evar_conv_x env isevars CONV) l1 l2))
-
- | IsMeta n, IsMeta m ->
- (n=m & (List.length(l1) = List.length(l2))
- & (List.for_all2 (evar_conv_x env isevars CONV) l1 l2))
-
- | IsSort s1, IsSort s2 when l1=[] & l2=[] -> base_sort_cmp pbty s1 s2
-
- | IsLambda (_,c1,c'1), IsLambda (_,c2,c'2) when l1=[] & l2=[] ->
- evar_conv_x env isevars CONV c1 c2
- & evar_conv_x env isevars CONV c'1 c'2
-
- | IsLetIn (_,b1,_,c'1), IsLetIn (_,b2,_,c'2) ->
- let f1 () =
- evar_conv_x env isevars CONV b1 b2
- & evar_conv_x env isevars pbty c'1 c'2
- & (List.length l1 = List.length l2)
- & (List.for_all2 (evar_conv_x env isevars CONV) l1 l2)
- and f2 () =
- evar_eqappr_x env isevars pbty (subst1 b1 c'1,l1) (subst1 b2 c'2,l2)
- in
- ise_try isevars [f1; f2]
-
- | IsLetIn (_,b1,_,c'1), _ -> (* On fait commuter les args avec le Let *)
- evar_eqappr_x env isevars pbty (subst1 b1 c'1,l1) appr2
-
- | _, IsLetIn (_,b2,_,c'2) ->
- evar_eqappr_x env isevars pbty appr1 (subst1 b2 c'2,l2)
-
- | IsProd (n,c1,c'1), IsProd (_,c2,c'2) when l1=[] & l2=[] ->
- evar_conv_x env isevars CONV c1 c2
- &
- (let d = nf_ise1 !isevars c1 in
- evar_conv_x (push_rel_assum (n,d) env) isevars pbty c'1 c'2)
-
- | IsMutInd (sp1,cl1), IsMutInd (sp2,cl2) ->
- sp1=sp2
- & array_for_all2 (evar_conv_x env isevars CONV) cl1 cl2
- & list_for_all2eq (evar_conv_x env isevars CONV) l1 l2
+ | Rigid c1, Rigid c2 -> match kind_of_term c1, kind_of_term c2 with
+
+ | IsCast (c1,_), _ -> evar_eqappr_x env isevars pbty (c1,l1) appr2
+
+ | _, IsCast (c2,_) -> evar_eqappr_x env isevars pbty appr1 (c2,l2)
+
+ | IsSort s1, IsSort s2 when l1=[] & l2=[] -> base_sort_cmp pbty s1 s2
+
+ | IsLambda (_,c1,c'1), IsLambda (_,c2,c'2) when l1=[] & l2=[] ->
+ evar_conv_x env isevars CONV c1 c2
+ & evar_conv_x env isevars CONV c'1 c'2
+
+ | IsLetIn (_,b1,_,c'1), IsLetIn (_,b2,_,c'2) ->
+ let f1 () =
+ evar_conv_x env isevars CONV b1 b2
+ & evar_conv_x env isevars pbty c'1 c'2
+ & (List.length l1 = List.length l2)
+ & (List.for_all2 (evar_conv_x env isevars CONV) l1 l2)
+ and f2 () =
+ evar_eqappr_x env isevars pbty (subst1 b1 c'1,l1)
+ (subst1 b2 c'2,l2)
+ in
+ ise_try isevars [f1; f2]
+
+ | IsLetIn (_,b1,_,c'1), _ ->(* On fait commuter les args avec le Let *)
+ evar_eqappr_x env isevars pbty (subst1 b1 c'1,l1) appr2
+
+ | _, IsLetIn (_,b2,_,c'2) ->
+ evar_eqappr_x env isevars pbty appr1 (subst1 b2 c'2,l2)
+
+ | IsProd (n,c1,c'1), IsProd (_,c2,c'2) when l1=[] & l2=[] ->
+ evar_conv_x env isevars CONV c1 c2
+ &
+ (let d = nf_ise1 !isevars c1 in
+ evar_conv_x (push_rel_assum (n,d) env) isevars pbty c'1 c'2)
+
+ | IsMutInd (sp1,cl1), IsMutInd (sp2,cl2) ->
+ sp1=sp2
+ & array_for_all2 (evar_conv_x env isevars CONV) cl1 cl2
+ & list_for_all2eq (evar_conv_x env isevars CONV) l1 l2
- | IsMutConstruct (sp1,cl1), IsMutConstruct (sp2,cl2) ->
- sp1=sp2
- & array_for_all2 (evar_conv_x env isevars CONV) cl1 cl2
- & list_for_all2eq (evar_conv_x env isevars CONV) l1 l2
-
- | IsMutCase (_,p1,c1,cl1), IsMutCase (_,p2,c2,cl2) ->
- evar_conv_x env isevars CONV p1 p2
- & evar_conv_x env isevars CONV c1 c2
- & (array_for_all2 (evar_conv_x env isevars CONV) cl1 cl2)
- & (list_for_all2eq (evar_conv_x env isevars CONV) l1 l2)
-
- | IsFix (li1,(tys1,_,bds1)), IsFix (li2,(tys2,_,bds2)) ->
- li1=li2
- & (array_for_all2 (evar_conv_x env isevars CONV) tys1 tys2)
- & (array_for_all2 (evar_conv_x env isevars CONV) bds1 bds2)
- & (list_for_all2eq (evar_conv_x env isevars CONV) l1 l2)
+ | IsMutConstruct (sp1,cl1), IsMutConstruct (sp2,cl2) ->
+ sp1=sp2
+ & array_for_all2 (evar_conv_x env isevars CONV) cl1 cl2
+ & list_for_all2eq (evar_conv_x env isevars CONV) l1 l2
+
+ | IsMutCase (_,p1,c1,cl1), IsMutCase (_,p2,c2,cl2) ->
+ evar_conv_x env isevars CONV p1 p2
+ & evar_conv_x env isevars CONV c1 c2
+ & (array_for_all2 (evar_conv_x env isevars CONV) cl1 cl2)
+ & (list_for_all2eq (evar_conv_x env isevars CONV) l1 l2)
+
+ | IsFix (li1,(tys1,_,bds1)), IsFix (li2,(tys2,_,bds2)) ->
+ li1=li2
+ & (array_for_all2 (evar_conv_x env isevars CONV) tys1 tys2)
+ & (array_for_all2 (evar_conv_x env isevars CONV) bds1 bds2)
+ & (list_for_all2eq (evar_conv_x env isevars CONV) l1 l2)
- | IsCoFix (i1,(tys1,_,bds1)), IsCoFix (i2,(tys2,_,bds2)) ->
- i1=i2
- & (array_for_all2 (evar_conv_x env isevars CONV) tys1 tys2)
- & (array_for_all2 (evar_conv_x env isevars CONV) bds1 bds2)
- & (list_for_all2eq (evar_conv_x env isevars CONV) l1 l2)
+ | IsCoFix (i1,(tys1,_,bds1)), IsCoFix (i2,(tys2,_,bds2)) ->
+ i1=i2
+ & (array_for_all2 (evar_conv_x env isevars CONV) tys1 tys2)
+ & (array_for_all2 (evar_conv_x env isevars CONV) bds1 bds2)
+ & (list_for_all2eq (evar_conv_x env isevars CONV) l1 l2)
- | (IsRel _ | IsVar _ | IsMeta _ | IsXtra _ | IsLambda _), _ -> false
- | _, (IsRel _ | IsVar _ | IsMeta _ | IsXtra _ | IsLambda _) -> false
+ | (IsMeta _ | IsXtra _ | IsLambda _), _ -> false
+ | _, (IsMeta _ | IsXtra _ | IsLambda _) -> false
- | (IsMutInd _ | IsMutConstruct _ | IsSort _ | IsProd _), _ -> false
- | _, (IsMutInd _ | IsMutConstruct _ | IsSort _ | IsProd _) -> false
+ | (IsMutInd _ | IsMutConstruct _ | IsSort _ | IsProd _), _ -> false
+ | _, (IsMutInd _ | IsMutConstruct _ | IsSort _ | IsProd _) -> false
- | (IsApp _ | IsMutCase _ | IsFix _ | IsCoFix _),
- (IsApp _ | IsMutCase _ | IsFix _ | IsCoFix _) -> false
+ | (IsApp _ | IsMutCase _ | IsFix _ | IsCoFix _),
+ (IsApp _ | IsMutCase _ | IsFix _ | IsCoFix _) -> false
+ | (IsRel _ | IsVar _ | IsConst _ | IsEvar _), _ -> assert false
+ | _, (IsRel _ | IsVar _ | IsConst _ | IsEvar _) -> assert false
and conv_record env isevars (c,bs,(xs,xs1),(us,us1),(ts,ts1),t) =