aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-12-19 09:14:42 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-12-19 09:14:42 +0000
commit5ad859d36a38b05bf2700a9507bd61e8a8964a53 (patch)
tree8cbd6aaba5eb1527cf520c679baae1d9156b00e1 /test-suite/success
parentd2f8cbfba4a1d5f9a2619ca83a26e315ebf71bfc (diff)
NatRing (2ème)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2326 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success')
-rw-r--r--test-suite/success/NatRing.v7
1 files changed, 6 insertions, 1 deletions
diff --git a/test-suite/success/NatRing.v b/test-suite/success/NatRing.v
index 47d9f9b5a..6a1eeccc6 100644
--- a/test-suite/success/NatRing.v
+++ b/test-suite/success/NatRing.v
@@ -1,5 +1,10 @@
Require ArithRing.
-Goal (S (S O))=(plus (S O) (S O)).
+Lemma l1 : (S (S O))=(plus (S O) (S O)).
NatRing.
Qed.
+
+Lemma l2 : (x:nat)(S (S x))=(plus (S O) (S x)).
+Intro.
+NatRing.
+Qed. \ No newline at end of file