aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/MSets/MSetList.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/MSetList.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/MSetList.v')
-rw-r--r--theories/MSets/MSetList.v32
1 files changed, 16 insertions, 16 deletions
diff --git a/theories/MSets/MSetList.v b/theories/MSets/MSetList.v
index b73af8f1a..45278eaf6 100644
--- a/theories/MSets/MSetList.v
+++ b/theories/MSets/MSetList.v
@@ -328,9 +328,9 @@ Module MakeRaw (X: OrderedType) <: RawSets X.
Qed.
Hint Resolve add_inf.
- Global Instance add_ok s x `(Ok s) : Ok (add x s).
+ Global Instance add_ok s x : forall `(Ok s), Ok (add x s).
Proof.
- intros s x; repeat rewrite <- isok_iff; revert s x.
+ repeat rewrite <- isok_iff; revert s x.
simple induction s; simpl.
intuition.
intros; elim_compare x a; inv; auto.
@@ -356,9 +356,9 @@ Module MakeRaw (X: OrderedType) <: RawSets X.
Qed.
Hint Resolve remove_inf.
- Global Instance remove_ok s x `(Ok s) : Ok (remove x s).
+ Global Instance remove_ok s x : forall `(Ok s), Ok (remove x s).
Proof.
- intros s x; repeat rewrite <- isok_iff; revert s x.
+ repeat rewrite <- isok_iff; revert s x.
induction s; simpl.
intuition.
intros; elim_compare x a; inv; auto.
@@ -399,9 +399,9 @@ Module MakeRaw (X: OrderedType) <: RawSets X.
Qed.
Hint Resolve union_inf.
- Global Instance union_ok s s' `(Ok s, Ok s') : Ok (union s s').
+ Global Instance union_ok s s' : forall `(Ok s, Ok s'), Ok (union s s').
Proof.
- intros s s'; repeat rewrite <- isok_iff; revert s s'.
+ repeat rewrite <- isok_iff; revert s s'.
induction2; constructors; try apply @ok; auto.
apply Inf_eq with x'; auto; apply union_inf; auto; apply Inf_eq with x; auto.
change (Inf x' (union (x :: l) l')); auto.
@@ -426,9 +426,9 @@ Module MakeRaw (X: OrderedType) <: RawSets X.
Qed.
Hint Resolve inter_inf.
- Global Instance inter_ok s s' `(Ok s, Ok s') : Ok (inter s s').
+ Global Instance inter_ok s s' : forall `(Ok s, Ok s'), Ok (inter s s').
Proof.
- intros s s'; repeat rewrite <- isok_iff; revert s s'.
+ repeat rewrite <- isok_iff; revert s s'.
induction2.
constructors; auto.
apply Inf_eq with x'; auto; apply inter_inf; auto; apply Inf_eq with x; auto.
@@ -457,9 +457,9 @@ Module MakeRaw (X: OrderedType) <: RawSets X.
Qed.
Hint Resolve diff_inf.
- Global Instance diff_ok s s' `(Ok s, Ok s') : Ok (diff s s').
+ Global Instance diff_ok s s' : forall `(Ok s, Ok s'), Ok (diff s s').
Proof.
- intros s s'; repeat rewrite <- isok_iff; revert s s'.
+ repeat rewrite <- isok_iff; revert s s'.
induction2.
Qed.
@@ -644,9 +644,9 @@ Module MakeRaw (X: OrderedType) <: RawSets X.
apply Inf_lt with x; auto.
Qed.
- Global Instance filter_ok s f `(Ok s) : Ok (filter f s).
+ Global Instance filter_ok s f : forall `(Ok s), Ok (filter f s).
Proof.
- intros s f; repeat rewrite <- isok_iff; revert s f.
+ repeat rewrite <- isok_iff; revert s f.
simple induction s; simpl.
auto.
intros x l Hrec f Hs; inv.
@@ -725,9 +725,9 @@ Module MakeRaw (X: OrderedType) <: RawSets X.
auto.
Qed.
- Global Instance partition_ok1 s f `(Ok s) : Ok (fst (partition f s)).
+ Global Instance partition_ok1 s f : forall `(Ok s), Ok (fst (partition f s)).
Proof.
- intros s f; repeat rewrite <- isok_iff; revert s f.
+ repeat rewrite <- isok_iff; revert s f.
simple induction s; simpl.
auto.
intros x l Hrec f Hs; inv.
@@ -735,9 +735,9 @@ Module MakeRaw (X: OrderedType) <: RawSets X.
case (f x); case (partition f l); simpl; auto.
Qed.
- Global Instance partition_ok2 s f `(Ok s) : Ok (snd (partition f s)).
+ Global Instance partition_ok2 s f : forall `(Ok s), Ok (snd (partition f s)).
Proof.
- intros s f; repeat rewrite <- isok_iff; revert s f.
+ repeat rewrite <- isok_iff; revert s f.
simple induction s; simpl.
auto.
intros x l Hrec f Hs; inv.