aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Sets
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-12-01 16:36:52 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-12-01 16:36:52 +0000
commitda882cfdac822da8d53e8c11b4a890e1643901ad (patch)
treee6cccb3c121feeefa0e26ef4b287fa334dbe5256 /theories/Sets
parent0780de3f579681aa80e5e353d3aaeeaa418f2369 (diff)
Fix make_exact_entry to allow applying [forall x, P x] hints directly,
avoiding the introduction of eta-redexes. Prioritize hints over intros in typeclass resolution to profit from that. Add a minor fix in coqdoc by F. Garillot. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12550 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Sets')
-rw-r--r--theories/Sets/Integers.v1
1 files changed, 0 insertions, 1 deletions
diff --git a/theories/Sets/Integers.v b/theories/Sets/Integers.v
index 443713211..01d3bda37 100644
--- a/theories/Sets/Integers.v
+++ b/theories/Sets/Integers.v
@@ -79,7 +79,6 @@ Section Integers_sect.
auto with sets arith.
apply Inhabited_intro with (x := 0).
apply Integers_defn.
- exact le_Order.
Defined.
Lemma le_total_order : Totally_ordered nat nat_po Integers.