aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init/Logic.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-02-10 08:44:40 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-02-10 08:44:40 +0000
commit5384ed9ab7557c515c8522b0229f10663e5a3161 (patch)
tree37a2a20ac67254049d9b8cf5159ad3f39ac054c5 /theories/Init/Logic.v
parent35e13590e82e5e3d2bc63e59c4fbedd1da2f66f4 (diff)
code mort
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@8022 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Init/Logic.v')
-rwxr-xr-xtheories/Init/Logic.v10
1 files changed, 0 insertions, 10 deletions
diff --git a/theories/Init/Logic.v b/theories/Init/Logic.v
index 7d9884505..cefbb989d 100755
--- a/theories/Init/Logic.v
+++ b/theories/Init/Logic.v
@@ -230,16 +230,6 @@ Section Logic_lemmas.
End equality.
-(* Is now a primitive principle
- Theorem eq_rect: (A:Type)(x:A)(P:A->Type)(P x)->(y:A)(eq ? x y)->(P y).
- Proof.
- Intros.
- Cut (identity A x y).
- NewDestruct 1; Auto.
- NewDestruct H; Auto.
- Qed.
-*)
-
Definition eq_ind_r :
forall (A:Type) (x:A) (P:A -> Prop), P x -> forall y:A, y = x -> P y.
intros A x P H y H0; elim sym_eq with (1 := H0); assumption.