aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Sorting/Sorting.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/Sorting/Sorting.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/Sorting/Sorting.v')
-rw-r--r--theories/Sorting/Sorting.v12
1 files changed, 3 insertions, 9 deletions
diff --git a/theories/Sorting/Sorting.v b/theories/Sorting/Sorting.v
index 06d35328b..77407c9ef 100644
--- a/theories/Sorting/Sorting.v
+++ b/theories/Sorting/Sorting.v
@@ -35,9 +35,7 @@ Hints Immediate eqA_dec leA_dec leA_antisym.
Local emptyBag := (EmptyBag A).
Local singletonBag := (SingletonBag eqA_dec).
-(************)
-(* lelistA *)
-(************)
+(** [lelistA] *)
Inductive lelistA [a:A] : (list A) -> Prop :=
nil_leA : (lelistA a (nil A))
@@ -50,9 +48,7 @@ Proof.
Intros; Inversion H; Trivial with datatypes.
Qed.
-(**************************************)
-(* definition for a list to be sorted *)
-(**************************************)
+(** definition for a list to be sorted *)
Inductive sort : (list A) -> Prop :=
nil_sort : (sort (nil A))
@@ -73,9 +69,7 @@ Induction y; Auto with datatypes.
Intros; Elim (!sort_inv a l); Auto with datatypes.
Qed.
-(****************************)
-(* merging two sorted lists *)
-(****************************)
+(** merging two sorted lists *)
Inductive merge_lem [l1:(list A);l2:(list A)] : Set :=
merge_exist : (l:(list A))(sort l) ->