aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/MSets/MSetWeakList.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-06-08 13:56:14 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-06-08 13:56:14 +0000
commitd14635b0c74012e464aad9e77aeeffda0f1ef154 (patch)
treebb913fa1399a1d4c7cdbd403e10c4efcc58fcdb1 /theories/MSets/MSetWeakList.v
parentf4c5934181c3e036cb77897ad8c8a192c999f6ad (diff)
Made option "Automatic Introduction" active by default before too many
people use the undocumented "Lemma foo x : t" feature in a way incompatible with this activation. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13090 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/MSets/MSetWeakList.v')
-rw-r--r--theories/MSets/MSetWeakList.v10
1 files changed, 5 insertions, 5 deletions
diff --git a/theories/MSets/MSetWeakList.v b/theories/MSets/MSetWeakList.v
index 8239ecef8..799e5f57e 100644
--- a/theories/MSets/MSetWeakList.v
+++ b/theories/MSets/MSetWeakList.v
@@ -275,7 +275,7 @@ Module MakeRaw (X:DecidableType) <: WRawSets X.
reflexivity.
Qed.
- Global Instance union_ok s s' `(Ok s, Ok s') : Ok (union s s').
+ Global Instance union_ok : forall s s' `(Ok s, Ok s'), Ok (union s s').
Proof.
induction s; simpl; auto; intros; inv; unfold flip; auto with *.
Qed.
@@ -291,7 +291,7 @@ Module MakeRaw (X:DecidableType) <: WRawSets X.
Global Instance inter_ok s s' `(Ok s, Ok s') : Ok (inter s s').
Proof.
- unfold inter, fold, flip; intros s.
+ unfold inter, fold, flip.
set (acc := nil (A:=elt)).
assert (Hacc : Ok acc) by constructors.
clearbody acc; revert acc Hacc.
@@ -322,7 +322,7 @@ Module MakeRaw (X:DecidableType) <: WRawSets X.
rewrite H2, <- mem_spec in H3; auto. congruence.
Qed.
- Global Instance diff_ok s s' `(Ok s, Ok s') : Ok (diff s s').
+ Global Instance diff_ok : forall s s' `(Ok s, Ok s'), Ok (diff s s').
Proof.
unfold diff; intros s s'; revert s.
induction s'; simpl; unfold flip; auto; intros. inv; auto with *.
@@ -491,7 +491,7 @@ Module MakeRaw (X:DecidableType) <: WRawSets X.
inversion_clear H; auto.
Qed.
- Global Instance partition_ok1 s f `(Ok s) : Ok (fst (partition f s)).
+ Global Instance partition_ok1 : forall s f `(Ok s), Ok (fst (partition f s)).
Proof.
simple induction s; simpl.
auto.
@@ -501,7 +501,7 @@ Module MakeRaw (X:DecidableType) <: WRawSets X.
case (f x); case (partition f l); simpl; constructors; auto.
Qed.
- Global Instance partition_ok2 s f `(Ok s) : Ok (snd (partition f s)).
+ Global Instance partition_ok2 : forall s f `(Ok s), Ok (snd (partition f s)).
Proof.
simple induction s; simpl.
auto.