aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init/Datatypes.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-09-11 19:56:40 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-09-11 19:56:40 +0000
commit753f8765dec057f24238e1d039504f92e503386a (patch)
tree77fc32b27596ffa40231ac9ad8f1dcf35cef53ed /theories/Init/Datatypes.v
parent33d4c7f37cb0ee1cec0214d30336334959f3d84e (diff)
Suppression notations redondantes en v8 : Fst, ProjS1, Value, Ex ...
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4353 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Init/Datatypes.v')
-rwxr-xr-xtheories/Init/Datatypes.v2
1 files changed, 2 insertions, 0 deletions
diff --git a/theories/Init/Datatypes.v b/theories/Init/Datatypes.v
index c0c999c4c..cb2c27284 100755
--- a/theories/Init/Datatypes.v
+++ b/theories/Init/Datatypes.v
@@ -74,8 +74,10 @@ Section projections.
Definition snd := [p:(prod A B)]Cases p of (pair x y) => y end.
End projections.
+V7only [
Notation Fst := (fst ? ?).
Notation Snd := (snd ? ?).
+].
Hints Resolve pair inl inr : core v62.