aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/MSets
diff options
context:
space:
mode:
Diffstat (limited to 'theories/MSets')
-rw-r--r--theories/MSets/MSetInterface.v5
-rw-r--r--theories/MSets/MSetList.v7
2 files changed, 4 insertions, 8 deletions
diff --git a/theories/MSets/MSetInterface.v b/theories/MSets/MSetInterface.v
index ae26fa7ed..10776a590 100644
--- a/theories/MSets/MSetInterface.v
+++ b/theories/MSets/MSetInterface.v
@@ -612,10 +612,7 @@ Module Raw2SetsOn (O:OrderedType)(M:RawSets O) <: SetsOn O.
Variable x y : elt.
Lemma compare_spec : CompSpec eq lt s s' (compare s s').
- Proof.
- assert (H:=@M.compare_spec s s' _ _).
- unfold compare; destruct M.compare; inversion_clear H; auto.
- Qed.
+ Proof. unfold compare; destruct (@M.compare_spec s s' _ _); auto. Qed.
(** Additional specification of [elements] *)
Lemma elements_spec2 : sort O.lt (elements s).
diff --git a/theories/MSets/MSetList.v b/theories/MSets/MSetList.v
index c29742332..d46803d75 100644
--- a/theories/MSets/MSetList.v
+++ b/theories/MSets/MSetList.v
@@ -805,10 +805,9 @@ Module MakeRaw (X: OrderedType) <: RawSets X.
CompSpec eq lt s s' (compare s s').
Proof.
intros s s' Hs Hs'.
- generalize (compare_spec_aux s s').
- destruct (compare s s'); inversion_clear 1; auto.
- apply CompLt. exists s, s'; repeat split; auto using @ok.
- apply CompGt. exists s', s; repeat split; auto using @ok.
+ destruct (compare_spec_aux s s'); constructor; auto.
+ exists s, s'; repeat split; auto using @ok.
+ exists s', s; repeat split; auto using @ok.
Qed.
End MakeRaw.