aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/univers.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2005-12-21 23:50:17 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2005-12-21 23:50:17 +0000
commit4d4f08acb5e5f56d38289e5629173bc1b8b5fd57 (patch)
treec160d442d54dbd15cbd0ab3500cdf94d0a6da74e /test-suite/success/univers.v
parent960859c0c10e029f9768d0d70addeca8f6b6d784 (diff)
Abandon tests syntaxe v7; remplacement des .v par des fichiers en syntaxe v8
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@7693 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success/univers.v')
-rw-r--r--test-suite/success/univers.v51
1 files changed, 26 insertions, 25 deletions
diff --git a/test-suite/success/univers.v b/test-suite/success/univers.v
index a2a1d0dd6..87edc4deb 100644
--- a/test-suite/success/univers.v
+++ b/test-suite/success/univers.v
@@ -1,41 +1,42 @@
(* This requires cumulativity *)
Definition Type2 := Type.
-Definition Type1 := Type : Type2.
+Definition Type1 : Type2 := Type.
-Lemma lem1 : (True->Type1)->Type2.
-Intro H.
-Apply H.
-Exact I.
+Lemma lem1 : (True -> Type1) -> Type2.
+intro H.
+apply H.
+exact I.
Qed.
-Lemma lem2 : (A:Type)(P:A->Type)(x:A)((y:A)(x==y)->(P y))->(P x).
-Auto.
+Lemma lem2 :
+ forall (A : Type) (P : A -> Type) (x : A),
+ (forall y : A, x = y -> P y) -> P x.
+auto.
Qed.
-Lemma lem3 : (P:Prop)P.
-Intro P ; Pattern P.
-Apply lem2.
+Lemma lem3 : forall P : Prop, P.
+intro P; pattern P in |- *.
+apply lem2.
Abort.
(* Check managing of universe constraints in inversion *)
(* Bug report #855 *)
-Inductive dep_eq : (X:Type) X -> X -> Prop :=
- | intro_eq : (X:Type) (f:X)(dep_eq X f f)
- | intro_feq : (A:Type) (B:A->Type)
- let T = (x:A)(B x) in
- (f, g:T) (x:A)
- (dep_eq (B x) (f x) (g x)) ->
- (dep_eq T f g).
+Inductive dep_eq : forall X : Type, X -> X -> Prop :=
+ | intro_eq : forall (X : Type) (f : X), dep_eq X f f
+ | intro_feq :
+ forall (A : Type) (B : A -> Type),
+ let T := forall x : A, B x in
+ forall (f g : T) (x : A), dep_eq (B x) (f x) (g x) -> dep_eq T f g.
Require Import Relations.
-Theorem dep_eq_trans : (X:Type) (transitive X (dep_eq X)).
+Theorem dep_eq_trans : forall X : Type, transitive X (dep_eq X).
Proof.
- Unfold transitive.
- Intros X f g h H1 H2.
- Inversion H1.
+ unfold transitive in |- *.
+ intros X f g h H1 H2.
+ inversion H1.
Abort.
@@ -50,8 +51,8 @@ Abort.
Especially, universe refreshing was not done for "set/pose" *)
-Lemma ind_unsec:(Q:nat->Type)True.
-Intro.
-Pose C:= (m:?)(Q m)->(Q m).
-Exact I.
+Lemma ind_unsec : forall Q : nat -> Type, True.
+intro.
+set (C := forall m, Q m -> Q m).
+exact I.
Qed.