aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/FSets/FSetRBT.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/FSets/FSetRBT.v')
-rw-r--r--theories/FSets/FSetRBT.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/theories/FSets/FSetRBT.v b/theories/FSets/FSetRBT.v
index 3ed463f1e..a3c378f0d 100644
--- a/theories/FSets/FSetRBT.v
+++ b/theories/FSets/FSetRBT.v
@@ -1,4 +1,4 @@
- (***********************************************************************)
+(***********************************************************************)
(* v * The Coq Proof Assistant / The Coq Development Team *)
(* <O___,, * INRIA-Rocquencourt & LRI-CNRS-Orsay *)
(* \VV/ *************************************************************)
@@ -52,7 +52,7 @@ Module Make [X : OrderedType] <: Sdep with Module E := X.
Hint In_tree := Constructors In_tree.
- (** [In_tree] is color-insensitive *)
+ (** [In_tree] is color-insensitive *)
Lemma In_color : (c,c':color)(x,y:elt)(l,r:tree)
(In_tree y (Node c l x r)) -> (In_tree y (Node c' l x r)).
@@ -303,7 +303,7 @@ Module Make [X : OrderedType] <: Sdep with Module E := X.
is_rbtree : (EX n:nat | (rbtree n the_tree)) }.
Definition t := t_.
- (** * Rotations *)
+ (** * Projections *)
Lemma t_is_bst : (s:t)(bst s).
Proof.