aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--kernel/environ.ml1
-rw-r--r--kernel/evd.ml2
-rw-r--r--kernel/evd.mli2
-rw-r--r--proofs/refiner.ml4
-rw-r--r--proofs/typing_ev.ml9
-rw-r--r--tactics/wcclausenv.ml2
-rw-r--r--tactics/wcclausenv.mli2
7 files changed, 11 insertions, 11 deletions
diff --git a/kernel/environ.ml b/kernel/environ.ml
index f715e985a..34261e735 100644
--- a/kernel/environ.ml
+++ b/kernel/environ.ml
@@ -43,7 +43,6 @@ let empty_env = {
let universes env = env.env_universes
let context env = env.env_context
-let metamap env = failwith "Environ.metamap: TODO: unifier metas et VE"
(* Construction functions. *)
diff --git a/kernel/evd.ml b/kernel/evd.ml
index b31f2f6b7..52e1a936e 100644
--- a/kernel/evd.ml
+++ b/kernel/evd.ml
@@ -65,6 +65,4 @@ let is_defined sigma ev =
let info = map sigma ev in
not (info.evar_body = Evar_empty)
-let metamap sigma = failwith "metamap : NOT YET IMPLEMENTED"
-
let evar_hyps ev = get_globals (context ev.evar_env)
diff --git a/kernel/evd.mli b/kernel/evd.mli
index 62378f921..2e55f578e 100644
--- a/kernel/evd.mli
+++ b/kernel/evd.mli
@@ -48,6 +48,4 @@ val is_evar : 'a evar_map -> evar -> bool
val is_defined : 'a evar_map -> evar -> bool
-val metamap : 'a evar_map -> (int * constr) list
-
val evar_hyps : 'a evar_info -> typed_type signature
diff --git a/proofs/refiner.ml b/proofs/refiner.ml
index 89aa18427..834ee6734 100644
--- a/proofs/refiner.ml
+++ b/proofs/refiner.ml
@@ -159,7 +159,7 @@ let refiner = function
subproof = Some hidden_proof;
ref = Some(r,spfl) }))
- | ((Context ctxt) as r) ->
+ | (Context ctxt) as r ->
(fun goal_sigma ->
let gl = goal_sigma.it in
let sg = mk_goal ctxt gl.evar_env gl.evar_concl in
@@ -174,7 +174,7 @@ let refiner = function
(* [Local_constraints lc] makes the local constraints be [lc] *)
- | ((Local_constraints lc) as r) ->
+ | (Local_constraints lc) as r ->
(fun goal_sigma ->
let gl = goal_sigma.it in
let ctxt = gl.evar_info in
diff --git a/proofs/typing_ev.ml b/proofs/typing_ev.ml
index 54a9d42dc..5e4815371 100644
--- a/proofs/typing_ev.ml
+++ b/proofs/typing_ev.ml
@@ -22,10 +22,13 @@ type 'a mach_flags = {
let rec execute mf env sigma cstr =
match kind_of_term cstr with
- | IsMeta _ ->
- anomaly "the kernel does not understand metas"
+ | IsMeta n ->
+ error "execute: found a non-instanciated goal"
+
| IsEvar _ ->
- anomaly "the kernel does not understand existential variables"
+ let ty = type_of_existential env sigma cstr in
+ let jty = execute mf env sigma ty in
+ { uj_val = cstr; uj_type = ty; uj_kind = jty.uj_type }
| IsRel n ->
relative env n
diff --git a/tactics/wcclausenv.ml b/tactics/wcclausenv.ml
index 44f17e816..e541c29db 100644
--- a/tactics/wcclausenv.ml
+++ b/tactics/wcclausenv.ml
@@ -19,6 +19,8 @@ open Clenv
write to Eduardo.Gimenez@inria.fr and ask for the prize :-)
-- Eduardo (11/8/97) *)
+type wc = walking_constraints
+
let pf_get_new_id id gls =
next_ident_away id (ids_of_sign (pf_untyped_hyps gls))
diff --git a/tactics/wcclausenv.mli b/tactics/wcclausenv.mli
index 8aee8dcb7..b1bf17e01 100644
--- a/tactics/wcclausenv.mli
+++ b/tactics/wcclausenv.mli
@@ -46,7 +46,7 @@ val res_pf_THEN_i :
(wc -> tactic) -> wc clausenv -> (wc clausenv -> int -> tactic) ->
int -> tactic
-val elim_res_pf_THEN_id :
+val elim_res_pf_THEN_i :
(wc -> tactic) -> wc clausenv -> (wc clausenv -> int -> tactic) ->
int -> tactic