aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/Rgeom.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/Reals/Rgeom.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/Reals/Rgeom.v')
-rw-r--r--theories/Reals/Rgeom.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/theories/Reals/Rgeom.v b/theories/Reals/Rgeom.v
index 55bdac0bf..c9fec070b 100644
--- a/theories/Reals/Rgeom.v
+++ b/theories/Reals/Rgeom.v
@@ -32,7 +32,7 @@ Intros; Unfold dist_euc; Apply Rsqr_incr_0; [Rewrite Rsqr_plus; Repeat Rewrite R
Save.
(******************************************************************)
-(* Translation *)
+(** Translation *)
(******************************************************************)
Definition xt[x,tx:R] : R := ``x+tx``.
@@ -47,7 +47,7 @@ Intros; Unfold Rsqr xt yt; Ring.
Save.
(******************************************************************)
-(* Rotation *)
+(** Rotation *)
(******************************************************************)
Definition xr [x,y,theta:R] : R := ``x*(cos theta)+y*(sin theta)``.
@@ -70,7 +70,7 @@ Unfold dist_euc; Intros; Apply Rsqr_inj; [Apply foo; Apply ge0_plus_ge0_is_ge0 |
Save.
(******************************************************************)
-(* Similarity *)
+(** Similarity *)
(******************************************************************)
Lemma isometric_rot_trans : (x1,y1,x2,y2,tx,ty,theta:R) ``(Rsqr (x1-x2))+(Rsqr (y1-y2)) == (Rsqr ((xr (xt x1 tx) (yt y1 ty) theta)-(xr (xt x2 tx) (yt y2 ty) theta))) + (Rsqr ((yr (xt x1 tx) (yt y1 ty) theta)-(yr (xt x2 tx) (yt y2 ty) theta)))``.