From d3950750f636057674c0ee527d5c05937faf90a2 Mon Sep 17 00:00:00 2001 From: herbelin Date: Sun, 19 Jan 2003 23:05:10 +0000 Subject: Il ne doit plus y avoir de preuves non terminées à la sortie du fichier MIME-Version: 1.0 Content-Type: text/plain; charset=UTF-8 Content-Transfer-Encoding: 8bit git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3538 85f007b7-540e-0410-9357-904b9bb8a0f7 --- test-suite/success/univers.v | 12 +++++++----- 1 file changed, 7 insertions(+), 5 deletions(-) (limited to 'test-suite/success/univers.v') diff --git a/test-suite/success/univers.v b/test-suite/success/univers.v index 28f9fe981..0a4b284f9 100644 --- a/test-suite/success/univers.v +++ b/test-suite/success/univers.v @@ -3,15 +3,17 @@ Definition Type2 := Type. Definition Type1 := Type : Type2. -Goal (True->Type1)->Type2. +Lemma lem1 : (True->Type1)->Type2. Intro H. Apply H. +Exact I. +Qed. -Lemma gg : (A:Type)(P:A->Type)(x:A)((y:A)(x==y)->(P y))->(P x). +Lemma lem2 : (A:Type)(P:A->Type)(x:A)((y:A)(x==y)->(P y))->(P x). Auto. Qed. -Lemma titi : (P:Prop)P. +Lemma lem3 : (P:Prop)P. Intro P ; Pattern P. -Apply gg. - +Apply lem2. +Abort. -- cgit v1.2.3