aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/output
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-04-27 22:13:04 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-04-27 22:13:04 +0200
commitc5b6321df0f83d6b29489bbddb920bdb1ebb96a8 (patch)
tree2f941e85d5cef3eba857291ed5ccf47d1385ed28 /test-suite/output
parent78c0afc1b292a196f33bce1e7e21ae83084f9b71 (diff)
Revert "A heuristic to add parentheses in the presence of rules such as"
Diffstat (limited to 'test-suite/output')
-rw-r--r--test-suite/output/Notations2.out4
-rw-r--r--test-suite/output/Notations2.v7
2 files changed, 0 insertions, 11 deletions
diff --git a/test-suite/output/Notations2.out b/test-suite/output/Notations2.out
index 593a5df84..6ff1d3837 100644
--- a/test-suite/output/Notations2.out
+++ b/test-suite/output/Notations2.out
@@ -54,7 +54,3 @@ end
: ∀ x : nat, x <= 0 -> {x0 : nat | x <= x0}
exist (Q x) y conj
: {x0 : A | Q x x0}
-fun x : nat => (## x) + x
- : nat -> nat
-fun x : nat => ## x + x
- : nat -> nat
diff --git a/test-suite/output/Notations2.v b/test-suite/output/Notations2.v
index d32758375..4e0d135d7 100644
--- a/test-suite/output/Notations2.v
+++ b/test-suite/output/Notations2.v
@@ -106,10 +106,3 @@ Check fun x (H:le x 0) => exist (le x) 0 H.
Parameters (A : Set) (x y : A) (Q : A -> A -> Prop) (conj : Q x y).
Check (exist (Q x) y conj).
-
-(* Check printing of notations that have arguments at higher level
- than the notation itself *)
-
-Notation "## a" := (S a) (at level 0, a at level 100).
-Check fun x => (S x) + x.
-Check fun x => S (x + x).