aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Structures
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-10-27 19:43:51 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-10-27 19:43:51 +0000
commit36c448f43c7fa16163b543b941be4a917a712a37 (patch)
tree73affd4fede1fea0dd56a2600bc420de769432e2 /theories/Structures
parent3178c7a29ff8b57a4598c4c5ded2eb29b8067dcf (diff)
Add a new vernacular command for controling implicit generalization of
variables with syntax: [Local?|Global] Generalizable Variable(s)? [all|none|id1 idn]. By default no variable is generalizable, so this patch breaks backward compatibility with files that used implicit generalization (through Instance declarations for example). To get back the old behavior, one just needs to use [Global Generalizable Variables all]. Make coq_makefile more robust using [mkdir -p]. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12428 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Structures')
-rw-r--r--theories/Structures/OrderedType2.v2
1 files changed, 2 insertions, 0 deletions
diff --git a/theories/Structures/OrderedType2.v b/theories/Structures/OrderedType2.v
index fdb1ccc24..c72d3a79d 100644
--- a/theories/Structures/OrderedType2.v
+++ b/theories/Structures/OrderedType2.v
@@ -270,6 +270,8 @@ Definition FstRel {A B}(R:relation A) : relation (A*B) :=
Definition SndRel {A B}(R:relation B) : relation (A*B) :=
fun p p' => R (snd p) (snd p').
+Generalizable Variables A B RA RB Ri Ro.
+
Instance ProdRel_equiv {A B} `(Equivalence A RA)`(Equivalence B RB) :
Equivalence (ProdRel RA RB).
Proof. firstorder. Qed.