aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init/Logic_Type.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-05-21 13:59:36 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-05-21 13:59:36 +0000
commit9e2ba1d42bfeff9aafc8384fb131330b725ce3be (patch)
tree5e4c6a613580cec0230ba83471686506352eaf1d /theories/Init/Logic_Type.v
parent6fe9381c21e6700791318920afd656a22c6a32b5 (diff)
Concentration des notations officielles dans Init/Notations; restructuration de Init
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4050 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Init/Logic_Type.v')
-rwxr-xr-xtheories/Init/Logic_Type.v26
1 files changed, 15 insertions, 11 deletions
diff --git a/theories/Init/Logic_Type.v b/theories/Init/Logic_Type.v
index 5ad3716ed..bdb3f687c 100755
--- a/theories/Init/Logic_Type.v
+++ b/theories/Init/Logic_Type.v
@@ -18,17 +18,20 @@ Require Export Logic.
Require LogicSyntax.
+(*
(** [allT A P], or simply [(ALLT x | P(x))], stands for [(x:A)(P x)]
when [A] is of type [Type] *)
-(*
Definition allT := [A:Type][P:A->Prop](x:A)(P x).
*)
V7only [
Syntactic Definition allT := all.
+Syntactic Definition inst := Logic.inst.
+Syntactic Definition gen := Logic.gen.
].
+(*
Section universal_quantification.
Variable A : Type.
@@ -45,7 +48,9 @@ Red; Auto.
Qed.
End universal_quantification.
+*)
+(*
(** * Existential Quantification *)
(** [exT A P], or simply [(EXT x | P(x))], stands for the existential
@@ -54,7 +59,6 @@ End universal_quantification.
(** [exT2 A P Q], or simply [(EXT x | P(x) & Q(x))], stands for the
existential quantification on both [P] and [Q] when [A] is of
type [Type] *)
-(*
Inductive exT [A:Type;P:A->Prop] : Prop
:= exT_intro : (x:A)(P x)->(exT A P).
*)
@@ -76,6 +80,7 @@ Syntactic Definition exT_intro2 := ex_intro2.
Syntactic Definition exT2_ind := ex2_ind.
].
+(*
(** Leibniz equality : [A:Type][x,y:A] (P:A->Prop)(P x)->(P y)
[eqT A x y], or simply [x==y], is Leibniz' equality when [A] is of
@@ -83,7 +88,6 @@ Syntactic Definition exT2_ind := ex2_ind.
symmetry, transitivity and stability by congruence *)
-(*
Inductive eqT [A:Type;x:A] : A -> Prop
:= refl_eqT : (eqT A x x).
@@ -107,22 +111,22 @@ Section Equality_is_a_congruence.
Lemma sym_eqT : (eqT ? x y) -> (eqT ? y x).
Proof.
- Induction 1; Trivial.
+ NewDestruct 1; Trivial.
Qed.
Lemma trans_eqT : (eqT ? x y) -> (eqT ? y z) -> (eqT ? x z).
Proof.
- Induction 2; Trivial.
+ NewDestruct 2; Trivial.
Qed.
Lemma congr_eqT : (eqT ? x y)->(eqT ? (f x) (f y)).
Proof.
- Induction 1; Trivial.
+ NewDestruct 1; Trivial.
Qed.
Lemma sym_not_eqT : ~(eqT ? x y) -> ~(eqT ? y x).
Proof.
- Red; Intros H H'; Apply H; Elim H'; Trivial.
+ Red; Intros H H'; Apply H; NewDestruct H'; Trivial.
Qed.
End Equality_is_a_congruence.
@@ -183,22 +187,22 @@ Section IdentityT_is_a_congruence.
Lemma sym_idT : (identityT ? x y) -> (identityT ? y x).
Proof.
- Induction 1; Trivial.
+ NewDestruct 1; Trivial.
Qed.
Lemma trans_idT : (identityT ? x y) -> (identityT ? y z) -> (identityT ? x z).
Proof.
- Induction 2; Trivial.
+ NewDestruct 2; Trivial.
Qed.
Lemma congr_idT : (identityT ? x y)->(identityT ? (f x) (f y)).
Proof.
- Induction 1; Trivial.
+ NewDestruct 1; Trivial.
Qed.
Lemma sym_not_idT : (notT (identityT ? x y)) -> (notT (identityT ? y x)).
Proof.
- Red; Intros H H'; Apply H; Elim H'; Trivial.
+ Red; Intros H H'; Apply H; NewDestruct H'; Trivial.
Qed.
End IdentityT_is_a_congruence.