aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rwxr-xr-xtheories/Init/Logic.v7
-rwxr-xr-xtheories7/Init/Logic.v6
2 files changed, 9 insertions, 4 deletions
diff --git a/theories/Init/Logic.v b/theories/Init/Logic.v
index e225bbddb..9e755c928 100755
--- a/theories/Init/Logic.v
+++ b/theories/Init/Logic.v
@@ -121,12 +121,15 @@ Definition all (A:Type) (P:A -> Prop) := forall x:A, P x.
Notation "'exists' x , p" := (ex (fun x => p))
(at level 200, x ident) : type_scope.
Notation "'exists' x : t , p" := (ex (fun x:t => p))
- (at level 200, x ident) : type_scope.
+ (at level 200, x ident, format "'exists' '/ ' x : t , '/ ' p")
+ : type_scope.
Notation "'exists2' x , p & q" := (ex2 (fun x => p) (fun x => q))
(at level 200, x ident, p at level 200) : type_scope.
Notation "'exists2' x : t , p & q" := (ex2 (fun x:t => p) (fun x:t => q))
- (at level 200, x ident, t at level 200, p at level 200) : type_scope.
+ (at level 200, x ident, t at level 200, p at level 200,
+ format "'exists2' '/ ' x : t , '/ ' '[' p & '/' q ']'")
+ : type_scope.
(** Universal quantification *)
diff --git a/theories7/Init/Logic.v b/theories7/Init/Logic.v
index 5881186de..ea8fb60ab 100755
--- a/theories7/Init/Logic.v
+++ b/theories7/Init/Logic.v
@@ -130,7 +130,8 @@ Notation "'EX' x | p" := (ex ? [x]p)
V8only "'exists' x , p" (at level 200, x ident, p at level 99).
Notation "'EX' x : t | p" := (ex ? [x:t]p)
(at level 10, p at level 8) : type_scope
- V8only "'exists' x : t , p" (at level 200, x ident, p at level 99).
+ V8only "'exists' x : t , p" (at level 200, x ident, p at level 99, format
+ "'exists' '/ ' x : t , '/ ' p").
V7only [ Notation Ex2 := (ex2 ?). ].
Notation "'EX' x | p & q" := (ex2 ? [x]p [x]q)
@@ -139,7 +140,8 @@ Notation "'EX' x | p & q" := (ex2 ? [x]p [x]q)
Notation "'EX' x : t | p & q" := (ex2 ? [x:t]p [x:t]q)
(at level 10, p, q at level 8) : type_scope
V8only "'exists2' x : t , p & q"
- (at level 200, x ident, t at level 200, p, q at level 99).
+ (at level 200, x ident, t at level 200, p, q at level 99, format
+ "'exists2' '/ ' x : t , '/ ' '[' p & '/' q ']'").
V7only [Notation All := (all ?).
Notation "'ALL' x | p" := (all ? [x]p)