aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/MSets/MSetAVL.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-06-15 17:03:30 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-06-15 17:03:30 +0000
commit412e75cda30682cf066974f7c80cb135b71ba90d (patch)
tree8c191d8b1ba9b2e24efb8b84605c694c07366d6b /theories/MSets/MSetAVL.v
parent4fcd729a1a123de61949d3dac659a39252625c0f (diff)
MSetAVL: for nicer extraction, we create only tree_ind, not tree_rect and tree_case
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13156 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/MSets/MSetAVL.v')
-rw-r--r--theories/MSets/MSetAVL.v5
1 files changed, 5 insertions, 0 deletions
diff --git a/theories/MSets/MSetAVL.v b/theories/MSets/MSetAVL.v
index d8486180c..6825e6881 100644
--- a/theories/MSets/MSetAVL.v
+++ b/theories/MSets/MSetAVL.v
@@ -35,6 +35,9 @@ Require Import MSetInterface ZArith Int.
Set Implicit Arguments.
Unset Strict Implicit.
+(* for nicer extraction, we create only logical inductive principles *)
+Local Unset Elimination Schemes.
+Local Unset Case Analysis Schemes.
(** * Ops : the pure functions *)
@@ -571,6 +574,8 @@ Module Import MX := OrderedTypeFacts X.
(** * Automation and dedicated tactics *)
+Scheme tree_ind := Induction for tree Sort Prop.
+
Local Hint Resolve MX.eq_refl MX.eq_trans MX.lt_trans @ok.
Local Hint Immediate MX.eq_sym.
Local Hint Unfold In lt_tree gt_tree.