From 27c28f38068b560882f2aaa9e147bfda54710504 Mon Sep 17 00:00:00 2001 From: herbelin Date: Mon, 22 Sep 2003 17:08:57 +0000 Subject: Système de renommage des noms de tactiques Ltac MIME-Version: 1.0 Content-Type: text/plain; charset=UTF-8 Content-Transfer-Encoding: 8bit git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4446 85f007b7-540e-0410-9357-904b9bb8a0f7 --- contrib/field/Field_Tactic.v | 1 + contrib/field/field.ml4 | 4 ++-- 2 files changed, 3 insertions(+), 2 deletions(-) (limited to 'contrib') diff --git a/contrib/field/Field_Tactic.v b/contrib/field/Field_Tactic.v index 1411c4a54..beb6d10ef 100644 --- a/contrib/field/Field_Tactic.v +++ b/contrib/field/Field_Tactic.v @@ -266,6 +266,7 @@ Recursive Tactic Definition Field_Gen_Aux FT := Tactic Definition Field_Gen FT := Unfolds FT;((InverseTest FT);Ring) Orelse (Field_Gen_Aux FT). +V7only [Tactic Definition field_gen := Field_Gen.]. (*****************************) (* Term Simplification *) diff --git a/contrib/field/field.ml4 b/contrib/field/field.ml4 index 57b8cd750..c5ec4df87 100644 --- a/contrib/field/field.ml4 +++ b/contrib/field/field.ml4 @@ -146,7 +146,7 @@ VERNAC COMMAND EXTEND Field (constr_of_opt a adiv_o) (constr_of rth) (constr_of ainv_l) ] END -(* Guesses the type and calls Field_Gen with the right theory *) +(* Guesses the type and calls field_gen with the right theory *) let field g = Library.check_required_library ["Coq";"field";"Field"]; let ist = { lfun=[]; debug=get_debug () } in @@ -156,7 +156,7 @@ let field g = | _ -> error "The statement is not built from Leibniz' equality" in let th = VConstr (lookup (pf_env g) typ) in (interp_tac_gen [(id_of_string "FT",th)] (get_debug ()) - <:tactic< match context with [|- (@eq _ _ _) ] => Field_Gen FT end >>) g + <:tactic< match context with [|- (@eq _ _ _) ] => field_gen FT end >>) g (* Verifies that all the terms have the same type and gives the right theory *) let guess_theory env evc = function -- cgit v1.2.3