aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Structures
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Structures')
-rw-r--r--theories/Structures/GenericMinMax.v14
-rw-r--r--theories/Structures/OrdersTac.v4
2 files changed, 9 insertions, 9 deletions
diff --git a/theories/Structures/GenericMinMax.v b/theories/Structures/GenericMinMax.v
index 01c6134b2..a62d96aa0 100644
--- a/theories/Structures/GenericMinMax.v
+++ b/theories/Structures/GenericMinMax.v
@@ -175,9 +175,6 @@ Qed.
(** *** Least-upper bound properties of [max] *)
-Definition max_l := max_l.
-Definition max_r := max_r.
-
Lemma le_max_l : forall n m, n <= max n m.
Proof.
intros; destruct (max_spec n m); intuition; order.
@@ -329,9 +326,6 @@ Proof. intros. symmetry; apply MPRev.max_assoc. Qed.
Lemma min_comm : forall n m, min n m == min m n.
Proof. intros. exact (MPRev.max_comm m n). Qed.
-Definition min_l := min_l.
-Definition min_r := min_r.
-
Lemma le_min_r : forall n m, min n m <= m.
Proof. intros. exact (MPRev.le_max_l m n). Qed.
@@ -544,6 +538,10 @@ Module MinMaxProperties (Import O:OrderedTypeFull')(Import M:HasMinMax O).
Module OT := OTF_to_TotalOrder O.
Include MinMaxLogicalProperties OT M.
Include MinMaxDecProperties O M.
+ Definition max_l := max_l.
+ Definition max_r := max_r.
+ Definition min_l := min_l.
+ Definition min_r := min_r.
Notation max_monotone := max_mono.
Notation min_monotone := min_mono.
Notation max_min_antimonotone := max_min_antimono.
@@ -611,6 +609,10 @@ Module UsualMinMaxProperties
Module OT := OTF_to_TotalOrder O.
Include UsualMinMaxLogicalProperties OT M.
Include UsualMinMaxDecProperties O M.
+ Definition max_l := max_l.
+ Definition max_r := max_r.
+ Definition min_l := min_l.
+ Definition min_r := min_r.
End UsualMinMaxProperties.
diff --git a/theories/Structures/OrdersTac.v b/theories/Structures/OrdersTac.v
index 64c764d9f..66a672c92 100644
--- a/theories/Structures/OrdersTac.v
+++ b/theories/Structures/OrdersTac.v
@@ -262,11 +262,9 @@ End OTF_to_OrderTac.
Module OT_to_OrderTac (OT:OrderedType).
Module OTF := OT_to_Full OT.
- Include !OTF_to_OrderTac OTF. (* Why a bang here ? *)
+ Include !OTF_to_OrderTac OTF.
End OT_to_OrderTac.
-
-
Module TotalOrderRev (O:TotalOrder) <: TotalOrder.
Definition t := O.t.