aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/output/Naming.out
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-12-02 21:41:06 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-12-02 21:41:06 +0000
commit4320ed3197791eda5dc29649c51dfa7f4e477c6b (patch)
tree36d809e06ee84a797aec7c30db37e548dac36509 /test-suite/output/Naming.out
parent3cb4411089c18351d57685f9abe455d3f61f308f (diff)
Continuing r12485-12486 and r12549 (cleaning around name generation)
- fixed misunderstanding of the role of nenv while simplifying code of occur_id in namegen.ml, - documented the possible incompatibilites in CHANGES - fixed output/Naming.v test, and fixed the count of misc. tests in test-suite/check. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12556 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/output/Naming.out')
-rw-r--r--test-suite/output/Naming.out36
1 files changed, 8 insertions, 28 deletions
diff --git a/test-suite/output/Naming.out b/test-suite/output/Naming.out
index 211a16714..86055c3ba 100644
--- a/test-suite/output/Naming.out
+++ b/test-suite/output/Naming.out
@@ -1,20 +1,9 @@
-Welcome to Coq localhost:/home/herbelin/coq/git,namegen (cd25d05cf1d1aa17f9c4f90d999559c2e7570b56)
-Parameter x2:nat.
-x2 is assumed
-Definition foo y := forall x x3 x4 S, x + S = x3 + x4 + y.
-foo is defined
-Section A.
-Variable x3:nat.
-x3 is assumed
-Goal forall x x1 x2 x3:nat,
- (forall x x3:nat, x+x1 = x2+x3) -> x+x1 = x2+x3.
1 subgoal
x3 : nat
============================
forall x x1 x4 x0 : nat,
- (forall x5 x6 : nat, x5 + x1 = x4 + x6) -> x + x1 = x4 + x0
-intros.
+ (forall x2 x5 : nat, x2 + x1 = x4 + x5) -> x + x1 = x4 + x0
1 subgoal
x3 : nat
@@ -25,30 +14,23 @@ intros.
H : forall x x3 : nat, x + x1 = x4 + x3
============================
x + x1 = x4 + x0
-Abort.
-Current goal aborted
-Goal forall x x1 x2 x3:nat,
- (forall x x3:nat, x+x1 = x2+x3 -> foo (S x + x1)) ->
- x+x1 = x2+x3 -> foo (S x).
1 subgoal
x3 : nat
============================
forall x x1 x4 x0 : nat,
- (forall x5 x6 : nat, x5 + x1 = x4 + x6 -> foo (S x5 + x1)) ->
+ (forall x2 x5 : nat, x2 + x1 = x4 + x5 -> foo (S x2 + x1)) ->
x + x1 = x4 + x0 -> foo (S x)
-unfold foo.
1 subgoal
x3 : nat
============================
forall x x1 x4 x0 : nat,
- (forall x5 x6 : nat,
- x5 + x1 = x4 + x6 ->
- forall x7 x8 x9 S : nat, x7 + S = x8 + x9 + (Datatypes.S x5 + x1)) ->
+ (forall x2 x5 : nat,
+ x2 + x1 = x4 + x5 ->
+ forall x6 x7 x8 S0 : nat, x6 + S0 = x7 + x8 + (S x2 + x1)) ->
x + x1 = x4 + x0 ->
forall x5 x6 x7 S : nat, x5 + S = x6 + x7 + Datatypes.S x
-do 4 intro.
1 subgoal
x3 : nat
@@ -57,12 +39,11 @@ do 4 intro.
x4 : nat
x0 : nat
============================
- (forall x5 x6 : nat,
- x5 + x1 = x4 + x6 ->
- forall x7 x8 x9 S : nat, x7 + S = x8 + x9 + (Datatypes.S x5 + x1)) ->
+ (forall x2 x5 : nat,
+ x2 + x1 = x4 + x5 ->
+ forall x6 x7 x8 S0 : nat, x6 + S0 = x7 + x8 + (S x2 + x1)) ->
x + x1 = x4 + x0 ->
forall x5 x6 x7 S : nat, x5 + S = x6 + x7 + Datatypes.S x
-do 2 intro.
1 subgoal
x3 : nat
@@ -76,7 +57,6 @@ do 2 intro.
H0 : x + x1 = x4 + x0
============================
forall x5 x6 x7 S : nat, x5 + S = x6 + x7 + Datatypes.S x
-do 4 intro.
1 subgoal
x3 : nat