aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Relations/Newman.v
diff options
context:
space:
mode:
authorGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-02-14 14:39:07 +0000
committerGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-02-14 14:39:07 +0000
commit67f72c93f5f364591224a86c52727867e02a8f71 (patch)
treeecf630daf8346e77e6620233d8f3e6c18a0c9b3c /theories/Relations/Newman.v
parentb239b208eb9a66037b0c629cf7ccb6e4b110636a (diff)
option -dump-glob pour coqdoc
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2474 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Relations/Newman.v')
-rwxr-xr-xtheories/Relations/Newman.v14
1 files changed, 7 insertions, 7 deletions
diff --git a/theories/Relations/Newman.v b/theories/Relations/Newman.v
index 2fe408543..57e93240a 100755
--- a/theories/Relations/Newman.v
+++ b/theories/Relations/Newman.v
@@ -26,12 +26,12 @@ Theorem coherence_intro : (x:A)(y:A)(z:A)(Rstar x z)->(Rstar y z)->(coherence x
Proof [x:A][y:A][z:A][h1:(Rstar x z)][h2:(Rstar y z)]
(exT_intro2 A (Rstar x) (Rstar y) z h1 h2).
-(* A very simple case of coherence : *)
+(** A very simple case of coherence : *)
Lemma Rstar_coherence : (x:A)(y:A)(Rstar x y)->(coherence x y).
Proof [x:A][y:A][h:(Rstar x y)](coherence_intro x y y h (Rstar_reflexive y)).
-(* coherence is symmetric *)
+(** coherence is symmetric *)
Lemma coherence_sym: (x:A)(y:A)(coherence x y)->(coherence y x).
Proof [x:A][y:A][h:(coherence x y)]
(exT2_ind A (Rstar x) (Rstar y) (coherence y x)
@@ -49,30 +49,30 @@ Definition noetherian :=
Section Newman_section.
-(* The general hypotheses of the theorem *)
+(** The general hypotheses of the theorem *)
Hypothesis Hyp1:noetherian.
Hypothesis Hyp2:(x:A)(local_confluence x).
-(* The induction hypothesis *)
+(** The induction hypothesis *)
Section Induct.
Variable x:A.
Hypothesis hyp_ind:(u:A)(R x u)->(confluence u).
-(* Confluence in x *)
+(** Confluence in [x] *)
Variables y,z:A.
Hypothesis h1:(Rstar x y).
Hypothesis h2:(Rstar x z).
-(* particular case x->u and u->*y *)
+(** particular case [x->u] and [u->*y] *)
Section Newman_.
Variable u:A.
Hypothesis t1:(R x u).
Hypothesis t2:(Rstar u y).
-(* In the usual diagram, we assume also x->v and v->*z *)
+(** In the usual diagram, we assume also [x->v] and [v->*z] *)
Theorem Diagram : (v:A)(u1:(R x v))(u2:(Rstar v z))(coherence y z).