aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-09-30 19:02:14 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-09-30 19:02:14 +0000
commitef5551e4ca73a93c0820f03ac702ee96e5e7b431 (patch)
tree570513e9aaf31ae7a6864a1dbc944aecec844124 /theories/Init
parent83015147aac453effee4d5b1b6363b31c56edd84 (diff)
Ajout infos de débogage de "universe inconsistency" quand option Set
Printing Universes est active. Ajout de l'option "using" à la tactique non documentée "auto decomp". Ajout de la base "extcore" pour étendre "auto decomp" avec des principes élémentaires tels que le dépliage de "iff". Quelques extensions/raffinements dans ChoiceFacts et ClassicalFacts. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10156 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Init')
-rw-r--r--theories/Init/Logic.v2
1 files changed, 2 insertions, 0 deletions
diff --git a/theories/Init/Logic.v b/theories/Init/Logic.v
index bdc8f9de6..8deb362cd 100644
--- a/theories/Init/Logic.v
+++ b/theories/Init/Logic.v
@@ -89,6 +89,8 @@ Theorem iff_sym : forall A B:Prop, (A <-> B) -> (B <-> A).
End Equivalence.
+Hint Unfold iff: extcore.
+
(** [(IF_then_else P Q R)], written [IF P then Q else R] denotes
either [P] and [Q], or [~P] and [Q] *)