aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init/Logic.v
diff options
context:
space:
mode:
authorGravatar pboutill <pboutill@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-04-12 20:49:11 +0000
committerGravatar pboutill <pboutill@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-04-12 20:49:11 +0000
commit3e70ea9c0967725bd320a6387d19cfb9d5a9b7fe (patch)
treed1804bed966aefae16dff65c41a27fa0ba5a9bce /theories/Init/Logic.v
parent8d0136caf2458c2a2457550b1af1299098b1d038 (diff)
"A -> B" is a notation for "forall _ : A, B".
No good reason for that except uniformity so revert this commit if you find a reason against it. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@15146 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Init/Logic.v')
-rw-r--r--theories/Init/Logic.v4
1 files changed, 3 insertions, 1 deletions
diff --git a/theories/Init/Logic.v b/theories/Init/Logic.v
index ca7d0073e..d391611dc 100644
--- a/theories/Init/Logic.v
+++ b/theories/Init/Logic.v
@@ -8,7 +8,9 @@
Set Implicit Arguments.
-Require Import Notations.
+Require Export Notations.
+
+Notation "A -> B" := (forall (_ : A), B) : type_scope.
(** * Propositional connectives *)