aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/tacinterp.ml
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-06-12 15:57:48 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-06-12 15:57:48 +0000
commit34e73d0e0e1e997a05307eaa2fab97d694271efa (patch)
treea400103c8612d5b51a79128820df9ec430ce4c4a /tactics/tacinterp.ml
parentf1dde2a39ea8230ab44eaa4ed4c69d716b64f0ce (diff)
Ajout option translate_syntax pour caractériser l'interprétation du traducteur à proprement parler
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4139 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tactics/tacinterp.ml')
-rw-r--r--tactics/tacinterp.ml5
1 files changed, 3 insertions, 2 deletions
diff --git a/tactics/tacinterp.ml b/tactics/tacinterp.ml
index e74405549..17b947ebd 100644
--- a/tactics/tacinterp.ml
+++ b/tactics/tacinterp.ml
@@ -642,8 +642,9 @@ and intern_tactic ist tac = (snd (intern_tactic_seq ist tac) : glob_tactic_expr)
and intern_tactic_seq ist = function
(* Traducteur v7->v8 *)
| TacAtom (_,TacReduce (Unfold [_,Ident (_,id)],_))
- when string_of_id id = "INZ" -> ist.ltacvars, TacId
-
+ when string_of_id id = "INZ" & !Options.translate_syntax
+ -> ist.ltacvars, TacId
+ (* Fin traducteur v7->v8 *)
| TacAtom (loc,t) ->
let lf = ref ist.ltacvars in