aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Logic/Eqdep_dec.v
diff options
context:
space:
mode:
authorGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-04-11 12:41:41 +0000
committerGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-04-11 12:41:41 +0000
commit4ac0580306ea9e45da1863316936d700969465ad (patch)
treebf7595cd76895f3a349e7e75ca9d64231b01dcf8 /theories/Logic/Eqdep_dec.v
parent8a7452976731275212f0c464385b380e2d590f5e (diff)
documentation automatique de la bibliothèque standard
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1578 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Logic/Eqdep_dec.v')
-rw-r--r--theories/Logic/Eqdep_dec.v10
1 files changed, 5 insertions, 5 deletions
diff --git a/theories/Logic/Eqdep_dec.v b/theories/Logic/Eqdep_dec.v
index 0b5c56ae1..a35993acd 100644
--- a/theories/Logic/Eqdep_dec.v
+++ b/theories/Logic/Eqdep_dec.v
@@ -8,14 +8,14 @@
(* $Id$ *)
-(* We prove that there is only one proof of x=x, i.e (refl_equal ? x).
- This holds if the equality upon the set of x is decidable.
+(* We prove that there is only one proof of [x=x], i.e [(refl_equal ? x)].
+ This holds if the equality upon the set of [x] is decidable.
A corollary of this theorem is the equality of the right projections
of two equal dependent pairs.
- Author: Thomas Kleymann <tms@dcs.ed.ac.uk> in Lego
+ Author: Thomas Kleymann \verb!<tms@dcs.ed.ac.uk>! in Lego
adapted to Coq by B. Barras
- Credit: Proofs up to K_dec follows an outline by Michael Hedberg
+ Credit: Proofs up to [K_dec] follows an outline by Michael Hedberg
*)
@@ -26,7 +26,7 @@ Scheme or_indd := Induction for or Sort Prop.
Implicit Arguments On.
- (* Bijection between eq and eqT *)
+ (* Bijection between [eq] and [eqT] *)
Definition eq2eqT: (A:Set)(x,y:A)x=y->x==y :=
[A,x,_,eqxy]<[y:A]x==y>Cases eqxy of refl_equal => (refl_eqT ? x) end.