aboutsummaryrefslogtreecommitdiffhomepage
path: root/kernel/mod_typing.ml
diff options
context:
space:
mode:
authorGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2014-02-24 20:46:32 +0100
committerGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2014-02-26 14:53:08 +0100
commit15b6c9b6fa268a9af6dd4f05961e469545e92a6f (patch)
tree2e5aacf72993b448d1e80b0cbfbf0a09091ecb32 /kernel/mod_typing.ml
parente6556db92d4c4fe9ba38f26b89f805095d2b2638 (diff)
Lazyconstr -> Opaqueproof
Make this module deal only with opaque proofs. Make discharging/substitution invariant more explicit via a third constructor.
Diffstat (limited to 'kernel/mod_typing.ml')
-rw-r--r--kernel/mod_typing.ml4
1 files changed, 2 insertions, 2 deletions
diff --git a/kernel/mod_typing.ml b/kernel/mod_typing.ml
index 6e656fad9..6c0f1b060 100644
--- a/kernel/mod_typing.ml
+++ b/kernel/mod_typing.ml
@@ -80,11 +80,11 @@ let rec check_with_def env struc (idl,c) mp equiv =
let cst = cb.const_constraints +++ cst1 +++ cst2 in
j.uj_val, cst
| Def cs ->
- let cst1 = Reduction.conv env' c (Lazyconstr.force cs) in
+ let cst1 = Reduction.conv env' c (Mod_subst.force_constr cs) in
let cst = cb.const_constraints +++ cst1 in
c, cst
in
- let def = Def (Lazyconstr.from_val c') in
+ let def = Def (Mod_subst.from_val c') in
let cb' =
{ cb with
const_body = def;