aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-05-21 22:43:42 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-05-21 22:43:42 +0000
commit17b2595145842b553c3daeb7eaf349526788723b (patch)
tree244cdea9aab4a3229b5f08d62395d7cfa004eb5c /contrib
parent4da48b01f420d8eccf6dcb2fea11bb4d9f8d8a86 (diff)
Suppression définitive de lmatch et or_metanum dans tacinterp
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4055 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'contrib')
-rw-r--r--contrib/correctness/ptactic.ml2
-rw-r--r--contrib/field/field.ml44
2 files changed, 3 insertions, 3 deletions
diff --git a/contrib/correctness/ptactic.ml b/contrib/correctness/ptactic.ml
index b272f6d04..dc7059413 100644
--- a/contrib/correctness/ptactic.ml
+++ b/contrib/correctness/ptactic.ml
@@ -69,7 +69,7 @@ let coqast_of_prog p =
(* 6. résolution implicites *)
deb_mess (fnl () ++ str"Resolution implicits (? => Meta(n))..." ++ fnl ());
- let oc = understand_gen_tcc Evd.empty (Global.env()) [] [] None r in
+ let oc = understand_gen_tcc Evd.empty (Global.env()) [] None r in
deb_print (Printer.prterm_env (Global.env())) (snd oc);
p,oc,ty,v
diff --git a/contrib/field/field.ml4 b/contrib/field/field.ml4
index 74fbd7f6b..36a29ab2d 100644
--- a/contrib/field/field.ml4
+++ b/contrib/field/field.ml4
@@ -144,13 +144,13 @@ END
(* Guesses the type and calls Field_Gen with the right theory *)
let field g =
Library.check_required_library ["Coq";"field";"Field"];
- let ist = { lfun=[]; lmatch=[]; debug=get_debug () } in
+ let ist = { lfun=[]; debug=get_debug () } in
let typ =
match Hipattern.match_with_equation (pf_concl g) with
| Some (eq,t::args) when eq = (Coqlib.build_coq_eq_data()).Coqlib.eq -> t
| _ -> error "The statement is not built from Leibniz' equality" in
let th = VConstr (lookup typ) in
- (interp_tac_gen [(id_of_string "FT",th)] [] (get_debug ())
+ (interp_tac_gen [(id_of_string "FT",th)] (get_debug ())
<:tactic< Match Context With [|-(!eq ?1 ?2 ?3)] -> Field_Gen FT>>) g
(* Verifies that all the terms have the same type and gives the right theory *)