aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Logic/Eqdep.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-01-27 14:37:30 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-01-27 14:37:30 +0000
commit40f6703ca86c6737d9d992154a2c879d722bb72e (patch)
treeb6aef293df45aaaa1acdf8cc27e69937d34c72ca /theories/Logic/Eqdep.v
parent20efeb644f65e3ddc866fd61979219b385aca0ab (diff)
MAJ simplification
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5254 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Logic/Eqdep.v')
-rwxr-xr-xtheories/Logic/Eqdep.v46
1 files changed, 22 insertions, 24 deletions
diff --git a/theories/Logic/Eqdep.v b/theories/Logic/Eqdep.v
index c5afa683a..9b379804d 100755
--- a/theories/Logic/Eqdep.v
+++ b/theories/Logic/Eqdep.v
@@ -16,7 +16,8 @@
- Invariance by Substitution of Reflexive Equality Proofs.
- Injectivity of Dependent Equality
- Uniqueness of Identity Proofs
- - Uniqueness of Reflexive Identity Proofs (usu. called Streicher's Axiom K)
+ - Uniqueness of Reflexive Identity Proofs
+ - Streicher's Axiom K
These statements are independent of the calculus of constructions [2].
@@ -43,7 +44,7 @@ Hint Constructors eq_dep: core v62.
Lemma eq_dep_sym :
forall (p q:U) (x:P p) (y:P q), eq_dep p x q y -> eq_dep q y p x.
Proof.
-simple induction 1; auto.
+destruct 1; auto.
Qed.
Hint Immediate eq_dep_sym: core v62.
@@ -51,46 +52,45 @@ Lemma eq_dep_trans :
forall (p q r:U) (x:P p) (y:P q) (z:P r),
eq_dep p x q y -> eq_dep q y r z -> eq_dep p x r z.
Proof.
-simple induction 1; auto.
+destruct 1; auto.
Qed.
+Scheme eq_indd := Induction for eq Sort Prop.
+
Inductive eq_dep1 (p:U) (x:P p) (q:U) (y:P q) : Prop :=
eq_dep1_intro : forall h:q = p, x = eq_rect q P y p h -> eq_dep1 p x q y.
-(** Invariance by Substitution of Reflexive Equality Proofs *)
-
-Axiom
- eq_rect_eq :
- forall (p:U) (Q:U -> Type) (x:Q p) (h:p = p), x = eq_rect p Q x p h.
-
Lemma eq_dep1_dep :
forall (p:U) (x:P p) (q:U) (y:P q), eq_dep1 p x q y -> eq_dep p x q y.
Proof.
-simple induction 1; intros eq_qp.
-cut (forall (h:q = p) (y0:P q), x = eq_rect q P y0 p h -> eq_dep p x q y0).
-intros; apply H0 with eq_qp; auto.
-rewrite eq_qp; intros h y0.
-elim eq_rect_eq.
-simple induction 1; auto.
+destruct 1 as (eq_qp, H).
+destruct eq_qp using eq_indd.
+rewrite H.
+apply eq_dep_intro.
Qed.
Lemma eq_dep_dep1 :
forall (p q:U) (x:P p) (y:P q), eq_dep p x q y -> eq_dep1 p x q y.
Proof.
-simple induction 1; intros.
+destruct 1.
apply eq_dep1_intro with (refl_equal p).
simpl in |- *; trivial.
Qed.
-Lemma eq_dep1_eq : forall (p:U) (x y:P p), eq_dep1 p x p y -> x = y.
-Proof.
-simple induction 1; intro.
-elim eq_rect_eq; auto.
-Qed.
+(** Invariance by Substitution of Reflexive Equality Proofs *)
+
+Axiom eq_rect_eq :
+ forall (p:U) (Q:U -> Type) (x:Q p) (h:p = p), x = eq_rect p Q x p h.
(** Injectivity of Dependent Equality is a consequence of *)
(** Invariance by Substitution of Reflexive Equality Proof *)
+Lemma eq_dep1_eq : forall (p:U) (x y:P p), eq_dep1 p x p y -> x = y.
+Proof.
+simple destruct 1; intro.
+rewrite <- eq_rect_eq; auto.
+Qed.
+
Lemma eq_dep_eq : forall (p:U) (x y:P p), eq_dep p x p y -> x = y.
Proof.
intros; apply eq_dep1_eq; apply eq_dep_dep1; trivial.
@@ -101,8 +101,6 @@ End Dependent_Equality.
(** Uniqueness of Identity Proofs (UIP) is a consequence of *)
(** Injectivity of Dependent Equality *)
-Scheme eq_indd := Induction for eq Sort Prop.
-
Lemma UIP : forall (U:Type) (x y:U) (p1 p2:x = y), p1 = p2.
Proof.
intros; apply eq_dep_eq with (P := fun y => x = y).
@@ -187,4 +185,4 @@ Qed.
Hint Resolve eq_dep_intro eq_dep_eq: core v62.
Hint Immediate eq_dep_sym: core v62.
-Hint Resolve inj_pair2 inj_pairT2: core. \ No newline at end of file
+Hint Resolve inj_pair2 inj_pairT2: core.