aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories7
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-02-28 13:03:01 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-02-28 13:03:01 +0000
commit9fcbb4ea786534982301f624d65e7d53e2f201be (patch)
tree036c8c4273b88a3ccbc9273cb4ebbd001cf222ff /theories7
parentdeef92a1e409e9c2b85fc2fa81ba03dcbbdc1f00 (diff)
MAJ Commentaires
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5397 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories7')
-rwxr-xr-xtheories7/Init/Logic.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories7/Init/Logic.v b/theories7/Init/Logic.v
index 84a545f3f..f21ac6131 100755
--- a/theories7/Init/Logic.v
+++ b/theories7/Init/Logic.v
@@ -121,7 +121,7 @@ Inductive ex2 [A:Type;P,Q:A->Prop] : Prop
Definition all := [A:Type][P:A->Prop](x:A)(P x).
-(*Rule order is important to give printing priority to fully typed ALL and EX*)
+(* Rule order is important to give printing priority to fully typed exists *)
V7only [ Notation Ex := (ex ?). ].
Notation "'EX' x | p" := (ex ? [x]p)