diff options
| author | herbelin | 2013-05-09 21:47:04 +0000 |
|---|---|---|
| committer | herbelin | 2013-05-09 21:47:04 +0000 |
| commit | 9f3ccbf420eec91410dea100b217a60f7defa5f2 (patch) | |
| tree | 7e218b44d609544e69ec6fe67ef5d5ae1d0e1c04 | |
| parent | 1eaebf4ab7616b2be16b957736e80f1d6100eae0 (diff) | |
Updating some output tests in test-suite:
InitSyntax, PrintInfos: consequence of r16467 which improved printing of sigT
Notations2: consequence of r16470 on using notations while asked to
print the body of an abbreviation
Notations: fix from r16417 was incomplete (and by the way associated
to a wrong commit message)
names: related to commit r16205 which aligned "In environment" with
the variables of the environment (maybe should it be better to still have
"In environment" printed after "Error: " but I don't know how to do
it with a forced newline).
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16503 85f007b7-540e-0410-9357-904b9bb8a0f7
| -rw-r--r-- | test-suite/output/InitSyntax.out | 2 | ||||
| -rw-r--r-- | test-suite/output/Notations.out | 6 | ||||
| -rw-r--r-- | test-suite/output/Notations2.out | 2 | ||||
| -rw-r--r-- | test-suite/output/PrintInfos.out | 6 | ||||
| -rw-r--r-- | test-suite/output/names.out | 3 |
5 files changed, 10 insertions, 9 deletions
diff --git a/test-suite/output/InitSyntax.out b/test-suite/output/InitSyntax.out index 55017469e7..bbfd3405af 100644 --- a/test-suite/output/InitSyntax.out +++ b/test-suite/output/InitSyntax.out @@ -1,5 +1,5 @@ Inductive sig2 (A : Type) (P Q : A -> Prop) : Type := - exist2 : forall x : A, P x -> Q x -> {x | P x & Q x} + exist2 : forall x : A, P x -> Q x -> {x : A | P x & Q x} For sig2: Argument A is implicit For exist2: Argument A is implicit diff --git a/test-suite/output/Notations.out b/test-suite/output/Notations.out index 37ce90af04..2fd5efe5d1 100644 --- a/test-suite/output/Notations.out +++ b/test-suite/output/Notations.out @@ -121,9 +121,9 @@ fun x : option Z => match x with end : option Z -> Z fun x : list ?103 => match x with - | NIL => NONE2 - | (_ :') t => SOME2 t - end + | NIL => NONE2 + | (_ :') t => SOME2 t + end : list ?103 -> option (list ?103) s : s diff --git a/test-suite/output/Notations2.out b/test-suite/output/Notations2.out index 3639c6c3de..b42ef2c511 100644 --- a/test-suite/output/Notations2.out +++ b/test-suite/output/Notations2.out @@ -38,7 +38,7 @@ let' f (x y : nat) (a:=0) (z : nat) (_ : bool) := x + y + z + 1 in f 0 1 2 : bool -> nat λ (f : nat -> nat) (x : nat), f(x) + S(x) : (nat -> nat) -> nat -> nat -Notation plus2 n := (S (S n)) +Notation plus2 n := (S(S(n))) λ n : list(nat), match n with | nil => 2 diff --git a/test-suite/output/PrintInfos.out b/test-suite/output/PrintInfos.out index 598bb72810..7bddcc6784 100644 --- a/test-suite/output/PrintInfos.out +++ b/test-suite/output/PrintInfos.out @@ -1,16 +1,16 @@ -existT : forall (A : Type) (P : A -> Type) (x : A), P x -> sigT P +existT : forall (A : Type) (P : A -> Type) (x : A), P x -> {x : A & P x} Argument A is implicit Argument scopes are [type_scope _ _ _] Expands to: Constructor Coq.Init.Specif.existT Inductive sigT (A : Type) (P : A -> Type) : Type := - existT : forall x : A, P x -> sigT P + existT : forall x : A, P x -> {x : A & P x} For sigT: Argument A is implicit For existT: Argument A is implicit For sigT: Argument scopes are [type_scope type_scope] For existT: Argument scopes are [type_scope _ _ _] -existT : forall (A : Type) (P : A -> Type) (x : A), P x -> sigT P +existT : forall (A : Type) (P : A -> Type) (x : A), P x -> {x : A & P x} Argument A is implicit Inductive eq (A : Type) (x : A) : A -> Prop := eq_refl : x = x diff --git a/test-suite/output/names.out b/test-suite/output/names.out index 1f13619cbf..ea7ce12662 100644 --- a/test-suite/output/names.out +++ b/test-suite/output/names.out @@ -1,5 +1,6 @@ The command has indeed failed with message: -=> Error: In environment +=> Error: + In environment y : nat The term "a y" has type "{y0 : nat | y = y0}" while it is expected to have type "{x : nat | x = y}". |
