diff options
author | Maxime Dénès <mail@maximedenes.fr> | 2017-05-23 09:13:12 +0200 |
---|---|---|
committer | Maxime Dénès <mail@maximedenes.fr> | 2017-05-23 09:13:12 +0200 |
commit | 884a70ba317a22f7fa5e84d19a88f345549c141e (patch) | |
tree | a51182be183ece2c6a6e4d9fc18ca259acae4b30 /test-suite/output | |
parent | 17e3f3b6a17145f7a51653de670263b7c3d613f3 (diff) | |
parent | ac333e6297bd7c32282fa5f47bebeb35826072df (diff) |
Merge PR#657: [test-suite] Add tests for goal printing.
Diffstat (limited to 'test-suite/output')
-rw-r--r-- | test-suite/output/goal_output.out | 8 | ||||
-rw-r--r-- | test-suite/output/goal_output.v | 13 |
2 files changed, 21 insertions, 0 deletions
diff --git a/test-suite/output/goal_output.out b/test-suite/output/goal_output.out new file mode 100644 index 000000000..773533a8d --- /dev/null +++ b/test-suite/output/goal_output.out @@ -0,0 +1,8 @@ +Nat.t = nat + : Set +Nat.t = nat + : Set +1 subgoal + + ============================ + False diff --git a/test-suite/output/goal_output.v b/test-suite/output/goal_output.v new file mode 100644 index 000000000..327b80b0a --- /dev/null +++ b/test-suite/output/goal_output.v @@ -0,0 +1,13 @@ +(* From + - https://coq.inria.fr/bugs/show_bug.cgi?id=5529 + - https://coq.inria.fr/bugs/show_bug.cgi?id=5537 + *) + +Print Nat.t. +Timeout 1 Print Nat.t. + +Lemma toto: False. +Set Printing All. +Show. +Abort. + |