aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib/fourier/fourierR.ml
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-12-09 08:40:00 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-12-09 08:40:00 +0000
commit18ffccadd1901e666ea3600263454446f52849d8 (patch)
treee7c69b9c82ba2e17ee52e5ff29632c817a76f7b7 /contrib/fourier/fourierR.ml
parentcd4d18cf0de8e8077a9c141a3e825b7647f03f8e (diff)
Ajout Simpl et Change sur des sous-termes
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3392 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'contrib/fourier/fourierR.ml')
-rw-r--r--contrib/fourier/fourierR.ml3
1 files changed, 2 insertions, 1 deletions
diff --git a/contrib/fourier/fourierR.ml b/contrib/fourier/fourierR.ml
index 1398499cf..9a2ff4d20 100644
--- a/contrib/fourier/fourierR.ml
+++ b/contrib/fourier/fourierR.ml
@@ -357,6 +357,7 @@ let my_cut c gl=
let concl = pf_concl gl in
apply_type (mkProd(Anonymous,c,concl)) [create_meta()] gl
;;
+
let exact = exact_check;;
let tac_use h = match h.htype with
@@ -522,7 +523,7 @@ let rec fourier gl=
else tac_zero_infeq_false gl (rational_to_fraction cres)
in
tac:=(tclTHENS (my_cut ineq)
- [tclTHEN (change_in_concl
+ [tclTHEN (change_in_concl None
(mkAppL [| parse "not"; ineq|]
))
(tclTHEN (apply (if sres then parse "Rnot_lt_lt"