aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/tauto.ml4
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-10-04 10:50:39 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-10-04 10:50:39 +0000
commit3b57619bd5dc164dcb51ad4fb390efd258940917 (patch)
treea86ebb8f52443374966b496de5b361166c4ed02d /tactics/tauto.ml4
parent88909c92cad0044dac83539b2b3d385242ed851e (diff)
Changed the way to support compatibility with previous versions.
Compatibility version is now a global parameter that every feature can individually browse. This avoids having to keep the names of options synchronous in their respective files and in now-removed file coqcompat.ml. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12372 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tactics/tauto.ml4')
-rw-r--r--tactics/tauto.ml44
1 files changed, 3 insertions, 1 deletions
diff --git a/tactics/tauto.ml4 b/tactics/tauto.ml4
index 6fea98377..60baa017c 100644
--- a/tactics/tauto.ml4
+++ b/tactics/tauto.ml4
@@ -49,6 +49,8 @@ let strict_unit = false
(* Whether inner iff are unfolded *)
let iff_unfolding = ref false
+let unfold_iff () = !iff_unfolding || Flags.version_less_or_equal Flags.V8_2
+
open Goptions
let _ =
declare_bool_option
@@ -256,7 +258,7 @@ let rec tauto_intuit t_reduce solver ist =
) >>
let reduction_not _ist =
- if !iff_unfolding then
+ if unfold_iff () then
<:tactic< unfold Coq.Init.Logic.not, Coq.Init.Logic.iff in * >>
else
<:tactic< unfold Coq.Init.Logic.not in * >>