aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Program/Syntax.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-07-22 21:06:23 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-07-22 21:06:23 +0000
commitf11fc1871babffd64e9d3be99197f91a0dfc8b69 (patch)
tree1e8f380abd19c027844d0291bdaa443a9aaf5f52 /theories/Program/Syntax.v
parentfc06cb87286e2b114c7f92500511d5914b8f7f48 (diff)
Made notations for exists, exists! and notations of Utf8.v recursive notations
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13317 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Program/Syntax.v')
-rw-r--r--theories/Program/Syntax.v9
1 files changed, 0 insertions, 9 deletions
diff --git a/theories/Program/Syntax.v b/theories/Program/Syntax.v
index 2c5fb79c5..bb52a0103 100644
--- a/theories/Program/Syntax.v
+++ b/theories/Program/Syntax.v
@@ -51,15 +51,6 @@ Implicit Arguments Vcons [[A] [n]].
(** Treating n-ary exists *)
-Notation " 'exists' x y , p" := (ex (fun x => (ex (fun y => p))))
- (at level 200, x ident, y ident, right associativity) : type_scope.
-
-Notation " 'exists' x y z , p" := (ex (fun x => (ex (fun y => (ex (fun z => p))))))
- (at level 200, x ident, y ident, z ident, right associativity) : type_scope.
-
-Notation " 'exists' x y z w , p" := (ex (fun x => (ex (fun y => (ex (fun z => (ex (fun w => p))))))))
- (at level 200, x ident, y ident, z ident, w ident, right associativity) : type_scope.
-
Tactic Notation "exists" constr(x) := exists x.
Tactic Notation "exists" constr(x) constr(y) := exists x ; exists y.
Tactic Notation "exists" constr(x) constr(y) constr(z) := exists x ; exists y ; exists z.