aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith/Zdiv.v
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-01-11 17:27:02 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-01-11 17:27:02 +0000
commite61dee5744110f9316305aeaa4c363af7655a989 (patch)
tree8cc0757d3ed2ad15bfec2441f9c0a07478dbc03d /theories/ZArith/Zdiv.v
parent6477ab0f7ea03a0563ca7ba2731d6aae1d3aa447 (diff)
Support "Local Obligation Tactic" (now the default in sections).
Update Numbers that was implicitely using [simpl_relation] instead of the default tactic [program_simpl]. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12647 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/ZArith/Zdiv.v')
-rw-r--r--theories/ZArith/Zdiv.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/theories/ZArith/Zdiv.v b/theories/ZArith/Zdiv.v
index a07b6d038..e9e963f97 100644
--- a/theories/ZArith/Zdiv.v
+++ b/theories/ZArith/Zdiv.v
@@ -306,6 +306,7 @@ Qed.
Module ZDiv <: ZDivFloor.ZDiv ZBinary.ZBinAxiomsMod.
Definition div := Zdiv.
Definition modulo := Zmod.
+ Local Obligation Tactic := simpl_relation.
Program Instance div_wd : Proper (eq==>eq==>eq) div.
Program Instance mod_wd : Proper (eq==>eq==>eq) modulo.