From 1826065d7603d0993b78829856a5725f253c782d Mon Sep 17 00:00:00 2001 From: letouzey Date: Fri, 12 Feb 2010 16:03:55 +0000 Subject: CompSpecType, a clone of CompSpec but in Type instead of Prop In interfaces fields like compare_spec, a CompSpec is prefered to get nice extraction, but then no "destruct (compare_spec .. ..)" is possible in a Type context. Now you can say there "destruct (CompSpec2Type (compare_spec ... ...))" This translate to the Type variant, and make the analysis on it (which is equivalent to analysing the comparison directly). git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12753 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/MSets/MSetInterface.v | 5 +---- 1 file changed, 1 insertion(+), 4 deletions(-) (limited to 'theories/MSets/MSetInterface.v') 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). -- cgit v1.2.3