aboutsummaryrefslogtreecommitdiff
path: root/kernel
diff options
context:
space:
mode:
authorcoq2002-08-13 14:44:24 +0000
committercoq2002-08-13 14:44:24 +0000
commita3848b0a10064fb7e206a503ac8b829cb9ce4666 (patch)
tree57715eb46564f71b91825c46ecb432a41c1ec095 /kernel
parentbc4e7b8c2317b2536eb42efb7cbf37d748ceb7c6 (diff)
Petites corrections ici et la
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2961 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'kernel')
-rw-r--r--kernel/subtyping.ml12
1 files changed, 12 insertions, 0 deletions
diff --git a/kernel/subtyping.ml b/kernel/subtyping.ml
index 5a7ce3cb32..4b4ae17cfd 100644
--- a/kernel/subtyping.ml
+++ b/kernel/subtyping.ml
@@ -145,6 +145,17 @@ let check_constant cst env msid1 l info1 cb2 spec2 =
| _ -> error ()
in
assert (cb1.const_hyps=[] && cb2.const_hyps=[]) ;
+ (*Start by checking bodies*)
+ match cb2.const_body with
+ | None -> check_conv cst conv_leq env cb1.const_type cb2.const_type
+ | Some c2 -> (* no checking types ! *)
+ let c1 = match cb1.const_body with
+ | None -> mkConst (make_kn (MPself msid1) empty_dirpath l)
+ | Some c1 -> c1
+ in
+ check_conv cst conv env c1 c2
+
+(* (*Start by checking types*)
let cst = check_conv cst conv_leq env cb1.const_type cb2.const_type in
match cb1.const_body, cb2.const_body with
| None, None -> cst
@@ -158,6 +169,7 @@ let check_constant cst env msid1 l info1 cb2 spec2 =
env
(mkConst (make_kn (MPself msid1) empty_dirpath l))
c2
+*)
let rec check_modules cst env msid1 l msb1 msb2 =
let cst = check_modtypes cst env (fst msb1) (fst msb2) false in