diff options
author | herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2006-01-19 09:18:59 +0000 |
---|---|---|
committer | herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2006-01-19 09:18:59 +0000 |
commit | b1ba21fe90b67abd052504075c9d0bc5ba6dded3 (patch) | |
tree | ce69ed943e0b16742e22fd200c3fe210865a9c14 /theories/Init | |
parent | e414b7ece0362fd9205cfee240141905c63af473 (diff) |
Correction associativité de IF et exists (visible à l'affichage uniquement à cause du traitement spécial du niveau binder_constr)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@7892 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Init')
-rwxr-xr-x | theories/Init/Logic.v | 11 |
1 files changed, 6 insertions, 5 deletions
diff --git a/theories/Init/Logic.v b/theories/Init/Logic.v index 3e3067c53..7d9884505 100755 --- a/theories/Init/Logic.v +++ b/theories/Init/Logic.v @@ -95,7 +95,7 @@ End Equivalence. Definition IF_then_else (P Q R:Prop) := P /\ Q \/ ~ P /\ R. Notation "'IF' c1 'then' c2 'else' c3" := (IF_then_else c1 c2 c3) - (at level 200) : type_scope. + (at level 200, right associativity) : type_scope. (** * First-order quantifiers *) @@ -128,15 +128,16 @@ Definition all (A:Type) (P:A -> Prop) := forall x:A, P x. (* Rule order is important to give printing priority to fully typed exists *) Notation "'exists' x , p" := (ex (fun x => p)) - (at level 200, x ident) : type_scope. + (at level 200, x ident, right associativity) : type_scope. Notation "'exists' x : t , p" := (ex (fun x:t => p)) - (at level 200, x ident, format "'[' 'exists' '/ ' x : t , '/ ' p ']'") + (at level 200, x ident, right associativity, + 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. + (at level 200, x ident, p at level 200, right associativity) : 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, + (at level 200, x ident, t at level 200, p at level 200, right associativity, format "'[' 'exists2' '/ ' x : t , '/ ' '[' p & '/' q ']' ']'") : type_scope. |