aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-10-10 20:50:04 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-10-10 20:50:04 +0000
commitec955042c050eb377fd5d46f95dafb36e5bd7d16 (patch)
treef0bed264c2b77739deba5cfaa1134fe761004c03 /theories/Init
parentfab4a88715538c7d302f0a3f0d185067f6d0d77e (diff)
identity est equivalent sur Type (sauf sans argument)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4590 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Init')
-rwxr-xr-xtheories/Init/Datatypes.v3
1 files changed, 1 insertions, 2 deletions
diff --git a/theories/Init/Datatypes.v b/theories/Init/Datatypes.v
index 2d35928c5..33eb6a322 100755
--- a/theories/Init/Datatypes.v
+++ b/theories/Init/Datatypes.v
@@ -42,7 +42,7 @@ Inductive Empty_set:Set :=.
member is the singleton datatype [identity A a a] whose
sole inhabitant is denoted [refl_identity A a] *)
-Inductive identity [A:Set; a:A] : A->Set :=
+Inductive identity [A:Type; a:A] : A->Set :=
refl_identity: (identity A a a).
Hints Resolve refl_identity : core v62.
@@ -77,7 +77,6 @@ V7only [
Notation Fst := (fst ? ?).
Notation Snd := (snd ? ?).
].
-
Hints Resolve pair inl inr : core v62.
V7only[