Library mathcomp.ssreflect.order

(* (c) Copyright 2006-2019 Microsoft Corporation and Inria.                  
 Distributed under the terms of CeCILL-B.                                  *)

From HB Require Import structures.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype ssrnat choice seq.
From mathcomp Require Import path fintype tuple bigop finset div prime finfun.
From mathcomp Require Import finset.

Types equipped with order relations NB: See CONTRIBUTING.md for an introduction to HB concepts and commands. This files defines types equipped with order relations.

How to use orders in MathComp?

Use one of the following modules implementing different theories (all located in the module Order): Order.LTheory: partially ordered types and lattices excluding complement and totality related theorems Order.CTheory: complemented lattices including Order.LTheory Order.TTheory: totally ordered types including Order.LTheory Order.Theory: ordered types including all of the above theory modules To access the definitions, notations, and the theory from, say, "Order.Xyz", insert "Import Order.Xyz." at the top of your scripts. In order to reason about abstract orders, notations are accessible by opening the scope "order_scope" bound to the delimiting key "O"; however, when dealing with another notation scope providing order notations for a concrete instance (e.g., "ring_scope"), it is not recommended to open "order_scope" at the same time.

Interfaces

Before providing the list of interfaces, a word is necessary about "displays". Each generic partial order has, as a first argument, a display to control the printing of notations. For example, when m and n are of type natdvd (an alias of nat), (Order.le m n) is displayed m %| n; natdvd is associated to the display dvd_display. Instantiating d with tt or an unknown display will lead to a default display for notations. See below for more details about displays. We provide the following interfaces for types equipped with an order: porderType d == the type of partially ordered types The HB class is called POrder. latticeType d == the type of non-distributive lattices The HB class is called Lattice. bPOrderType d == partial order with a bottom element The HB class is called BPOrder. bLatticeType d == latticeType with a bottom element The HB class is called BLattice. tPOrderType d == partial order with a top element The HB class is called TPOrder. tbPOrderType d == partial order with a top and a bottom elements The HB class is called TBPOrder. tLatticeType d == latticeType with a top element The HB class is called TLattice. tbLatticeType d == latticeType with both a top and a bottom The HB class is called TBLattice. distrLatticeType d == the type of distributive lattices The HB class is called DistrLattice. bDistrLatticeType d == distrLatticeType with a bottom element The HB class is called BDistrLattice. tbDistrLatticeType d == distrLatticeType with both a top and a bottom The HB class is called TBDistrLattice. cbDistrLatticeType d == the type of sectionally complemented distributive lattices (lattices with bottom and a difference operation) The HB class is called CBDistrLattice. ctbDistrLatticeType d == the type of complemented distributive lattices (lattices with top, bottom, difference, and complement) The HB class is called CTBDistrLattice. orderType d == the type of totally ordered types The HB class is called Total. finPOrderType d == the type of partially ordered finite types The HB class is called FinPOrder. finLatticeType d == the type of nonempty finite non-distributive lattices The HB class is called FinLattice. finDistrLatticeType d == the type of nonempty finite distributive lattices The HB class is called FinDistrLattice. finCDistrLatticeType d == the type of nonempty finite complemented distributive lattices The HB class is called FinCDistrLattice. finOrderType d == the type of nonempty totally ordered finite types The HB class is called FinTotal. and their joins with subType: subPOrder d T P d' == join of porderType d' and subType (P : pred T) such that val is monotonic The HB class is called SubPOrder. meetSubLattice d T P d' == join of latticeType d' and subType (P : pred T) such that val is monotonic and a morphism for meet The HB class is called MeetSubLattice. joinSubLattice d T P d' == join of latticeType d' and subType (P : pred T) such that val is monotonic and a morphism for join The HB class is called JoinSubLattice. subLattice d T P d' == join of JoinSubLattice and MeetSubLattice The HB class is called SubLattice. bJoinSubLattice d T P d' == join of JoinSubLattice and BLattice such that val is a morphism for \bot The HB class is called BJoinSubLattice. tMeetSubLattice d T P d' == join of MeetSubLattice and TLattice such that val is a morphism for \top The HB class is called TMeetSubLattice. bSubLattice d T P d' == join of SubLattice and BLattice such that val is a morphism for \bot The HB class is called BSubLattice. tSubLattice d T P d' == join of SubLattice and TLattice such that val is a morphism for \top The HB class is called BSubLattice. subOrder d T P d' == join of orderType d' and subLatticeType d T P d' The HB class is called SubOrder. subPOrderLattice d T P d' == join of SubPOrder and Lattice The HB class is called SubPOrderLattice. subPOrderBLattice d T P d' == join of SubPOrder and BLattice The HB class is called SubPOrderBLattice. subPOrderTLattice d T P d' == join of SubPOrder and TLattice The HB class is called SubPOrderTLattice. subPOrderTBLattice d T P d' == join of SubPOrder and TBLattice The HB class is called SubPOrderTBLattice. meetSubBLattice d T P d' == join of MeetSubLattice and BLattice The HB class is called MeetSubBLattice. meetSubTLattice d T P d' == join of MeetSubLattice and TLattice The HB class is called MeetSubTLattice. meetSubTBLattice d T P d' == join of MeetSubLattice and TBLattice The HB class is called MeetSubTBLattice. joinSubBLattice d T P d' == join of JoinSubLattice and BLattice The HB class is called JoinSubBLattice. joinSubTLattice d T P d' == join of JoinSubLattice and TLattice The HB class is called JoinSubTLattice. joinSubTBLattice d T P d' == join of JoinSubLattice and TBLattice The HB class is called JoinSubTBLattice. subBLattice d T P d' == join of SubLattice and BLattice The HB class is called SubBLattice. subTLattice d T P d' == join of SubLattice and TLattice The HB class is called SubTLattice. subTBLattice d T P d' == join of SubLattice and TBLattice The HB class is called SubTBLattice. bJoinSubTLattice d T P d' == join of BJoinSubLattice and TBLattice The HB class is called BJoinSubTLattice. tMeetSubBLattice d T P d' == join of TMeetSubLattice and TBLattice The HB class is called TMeetSubBLattice. bSubTLattice d T P d' == join of BSubLattice and TBLattice The HB class is called BSubTLattice. tSubBLattice d T P d' == join of TSubLattice and TBLattice The HB class is called TSubBLattice. tbSubBLattice d T P d' == join of BSubLattice and TSubLattice The HB class is called TBSubLattice. Morphisms between the above structures: OrderMorphism.type d T d' T' == monotonic function between the two porder := {omorphism T -> T'} MeetLatticeMorphism.type d T d' T', JoinLatticeMorphism.type d T d' T', LatticeMorphism.type d T d' T' == monotonic function between two lattices which are morphism for meet, join, and meet/join respectively BLatticeMorphism.type d T d' T' := {blmorphism T -> T'}, TLatticeMorphism.type d T d' T' := {tlmorphism T -> T'}, TBLatticeMorphism.type d T d' T' := {tblmorphism T -> T'} == monotonic function between two lattices with bottom/top which are morphism for bottom/top Closedness predicates for the algebraic structures: meetLatticeClosed d T == predicate closed under meet on T : latticeType d The HB class is MeetLatticeClosed. joinLatticeClosed d T == predicate closed under join on T : latticeType d The HB class is JoinLatticeClosed. latticeClosed d T == predicate closed under meet and join The HB class is JoinLatticeClosed. bLatticeClosed d T == predicate that contains bottom The HB class is BLatticeClosed. tLatticeClosed d T == predicate that contains top The HB class is TLatticeClosed. tbLatticeClosed d T == predicate that contains top and bottom the HB class ie TBLatticeClosed. bJoinLatticeClosed d T == predicate that contains bottom and is closed under join The HB class is BJoinLatticeClosed. tMeetLatticeClosed d T == predicate that contains top and is closed under meet The HB class is TMeetLatticeClosed.

Useful lemmas:

On orderType, leP ltP ltgtP are the three main lemmas for case analysis. On porderType, one may use comparableP, comparable_leP, comparable_ltP, and comparable_ltgtP, which are the four main lemmas for case analysis. For x, y of type T, where T is canonically a porderType d: x <= y <-> x is less than or equal to y x < y <-> x is less than y (:= (y != x) && (x <= y)) min x y <-> if x < y then x else y max x y <-> if x < y then y else x x >= y <-> x is greater than or equal to y (:= y <= x) x > y <-> x is greater than y (:= y < x) x <= y ?= iff C <-> x is less than y, or equal iff C is true x < y ?<= if C <-> x is smaller than y, and strictly if C is false x >=< y <-> x and y are comparable (:= (x <= y) || (y <= x)) x >< y <-> x and y are incomparable (:= ~~ x >=< y) f \min g <-> the function x |-> Order.min (f x) (g x); f \min g simplifies on application f \max g <-> the function x |-> Order.max (f x) (g x); f \max g simplifies on application For x, y of type T, where T is canonically a latticeType d: x `&` y == the meet of x and y x `|` y == the join of x and y In a type T, where T is canonically a bLatticeType d: \bot == the bottom element \join_<range> e == iterated join of a lattice with a bottom In a type T, where T is canonically a tbLatticeType d: \top == the top element \meet_<range> e == iterated meet of a lattice with a top For x, y of type T, where T is canonically a cbDistrLatticeType d: x `\` y == the (sectional) complement of y in [\bot, x] For x of type T, where T is canonically a ctbDistrLatticeType d: ~` x == the complement of x in [\bot, \top] There are three distinct uses of the symbols <, <=, >, >=, _ <= _ ?= iff _, >=<, and >< in the default display: they can be 0-ary, unary (prefix), and binary (infix). 0. <%O, <=%O, >%O, >=%O, <?=%O, >=<%O, and ><%O stand respectively for lt, le, gt, ge, leif (_ <= _ ?= iff _), comparable, and incomparable. 1. (< x), (<= x), (> x), (>= x), (>=< x), and (>< x) stand respectively for (>%O x), (>=%O x), (<%O x), (<=%O x), (>=<%O x), and (><%O x). So (< x) is a predicate characterizing elements smaller than x. 2. (x < y), (x <= y), ... mean what they are expected to. These conventions are compatible with Haskell's, where ((< y) x) = (x < y) = ((<) x y), except that we write <%O instead of (<). Like each generic partial order, lattice operations symbols also have a first argument which is the display (ranged over by d of type unit), the second which is the minimal structure they operate on and then the operands. Here is the exhaustive l list of all such symbols for partial orders and lattices together with their default printed notation (as displayed by Check). For porderType T (in function_scope): <=%O == @Order.le d T <%O == @Order.lt d T >=<%O == @Order.comparable d T >=%O == @Order.ge d T >%O == @Order.gt d T <?=%O == @Order.leif d T <?<=%O == @Order.lteif d T For latticeType T (in order_scope): x `&` y == @Order.meet d T x y x `|` y == @Order.join d T x y For bLatticeType T (in order_scope): \bot == @Order.bottom d T For tLatticeType T (in order_scope): \top == @Order.top d T For cbDistrLatticeType T (in order_scope): x `|` y == @Order.sub d T x y For ctbDistrLatticeType T (in order_scope): ~` x == @Order.compl d T x For porderType we provide the following operations: [arg min_(i < i0 | P) M] == a value i : T minimizing M : R, subject to the condition P (i may appear in P and M), and provided P holds for i0. [arg max_(i > i0 | P) M] == a value i maximizing M subject to P and provided P holds for i0. [arg min_(i < i0 in A) M] == an i \in A minimizing M if i0 \in A. [arg max_(i > i0 in A) M] == an i \in A maximizing M if i0 \in A. [arg min_(i < i0) M] == an i : T minimizing M, given i0 : T. [arg max_(i > i0) M] == an i : T maximizing M, given i0 : T. with head symbols Order.arg_min and Order.arg_max The user may use extremumP or extremum_inP to eliminate them.
  • > patterns for contextual rewriting: leLHS := (X in (X <= _)%O)%pattern leRHS := (X in (_ <= X)%O)%pattern ltLHS := (X in (X < _)%O)%pattern ltRHS := (X in (_ < X)%O)%pattern
One may use displays either for convenience or to disambiguate between different structures defined on "copies" of a type (as explained below). We provide the following "copies" of types: natdvd := nat == a "copy" of nat which is canonically ordered using divisibility predicate dvdn Notation %|, %<|, gcd, lcm are used instead of <=, <, meet and join. T^d := dual T, where dual is a new definition for (fun T => T) == a "copy" of T, such that if T is canonically ordered, then T^d is canonically ordered with the dual order, and displayed with an extra ^d in the notation i.e. <=^d, <^d, >=<^d, ><^d, `&`^d, `|`^d are used and displayed instead of <=, <, >=<, ><, `&`, `|` T *prod[d] T' := T * T' == a "copy" of the cartesian product such that, if T and T' are canonically ordered, then T *prod[d] T' is canonically ordered in product order, i.e., (x1, x2) <= (y1, y2) = (x1 <= y1) && (x2 <= y2), and displayed in display d T *p T' := T *prod[prod_display] T' where prod_display adds an extra ^p to all notations T *lexi[d] T' := T * T' == a "copy" of the cartesian product such that, if T and T' are canonically ordered, then T *lexi[d] T' is canonically ordered in lexicographic order, i.e., (x1, x2) <= (y1, y2) = (x1 <= y1) && ((x1 >= y1) ==> (x2 <= y2)) and (x1, x2) < (y1, y2) = (x1 <= y1) && ((x1 >= y1) ==> (x2 < y2)) and displayed in display d T *l T' := T *lexi[lexi_display] T' where lexi_display adds an extra ^l to all notations seqprod_with d T := seq T == a "copy" of seq, such that if T is canonically ordered, then seqprod_with d T is canonically ordered in product order, i.e., [:: x1, .., xn] <= [y1, .., yn] = (x1 <= y1) && ... && (xn <= yn) and displayed in display d n.-tupleprod[d] T == same with n.tuple T seqprod T := seqprod_with prod_display T n.-tupleprod T := n.-tuple[prod_display] T seqlexi_with d T := seq T == a "copy" of seq, such that if T is canonically ordered, then seqprod_with d T is canonically ordered in lexicographic order, i.e., [:: x1, .., xn] <= [y1, .., yn] = (x1 <= x2) && ((x1 >= y1) ==> ((x2 <= y2) && ...)) and displayed in display d n.-tuplelexi[d] T == same with n.tuple T seqlexi T := lexiprod_with lexi_display T n.-tuplelexi T := n.-tuple[lexi_display] T {subset[d] T} := {set T} == a "copy" of set which is canonically ordered by the subset order and displayed in display d {subset T} := {subset[subset_display] T} Existing displays are either dual_display d (where d is a display), dvd_display, ring_display (from algebra/ssrnum.v to change the scope of the usual notations to ring_scope). We also provide lexi_display and prod_display for lexicographic and product order respectively. Beware of the asymmetry of canonical structure inference. Canonical structure inference makes it possible to infer the display associated to a type (or a named copy of a type) from the name. However, it does not help finding the named copy when the display is provided. In this sense displays are merely used to inform the user and the notation mechanism of what the inference did; they are not additional input for the inference. Alternative notation displays can be defined by : 1. declaring a new opaque definition of type unit. Using the idiom `Fact my_display : unit. Proof. exact: tt. Qed.` 2. using this symbol to tag canonical porderType structures using `HB.instance Definition _ := isPOrder.Build my_display my_type ...`, 3. declaring notations for the main operations of this library, by setting the first argument of the definition to the display, e.g. `Notation my_syndef_le x y := @Order.le my_display _ x y.` or `Notation "x <=< y" := @Order.lt my_display _ x y (at level ...).` Non overloaded notations will default to the default display. We suggest the user to refer to the example of natdvd (further explained below) as guide line example to add their own displays. The following notations are provided to build substructures: [SubChoice_isSubPOrder of U by <: with disp] == [SubChoice_isSubPOrder of U by <: ] == porderType mixin for a subType whose base type is a porderType [SubPOrder_isSubLattice of U by <: with disp] == [SubPOrder_isSubLattice of U by <: ] == [SubChoice_isSubLattice of U by <: with disp] == [SubChoice_isSubLattice of U by <: ] == latticeType mixin for a subType whose base type is a latticeType and whose predicate's is a latticeClosed [SubPOrder_isBSubLattice of U by <: with disp] == [SubPOrder_isBSubLattice of U by <: ] == [SubChoice_isBSubLattice of U by <: with disp] == [SubChoice_isBSubLattice of U by <: ] == blatticeType mixin for a subType whose base type is a blatticeType and whose predicate's is both a latticeClosed and a bLatticeClosed [SubPOrder_isTSubLattice of U by <: with disp] == [SubPOrder_isTSubLattice of U by <: ] == [SubChoice_isTSubLattice of U by <: with disp] == [SubChoice_isTSubLattice of U by <: ] == tlatticeType mixin for a subType whose base type is a tlatticeType and whose predicate's is both a latticeClosed and a tLatticeClosed [SubPOrder_isTBSubLattice of U by <: with disp] == [SubPOrder_isTBSubLattice of U by <: ] == [SubChoice_isTBSubLattice of U by <: with disp] == [SubChoice_isTBSubLattice of U by <: ] == tblatticeType mixin for a subType whose base type is a tblatticeType and whose predicate's is both a latticeClosed and a tbLatticeClosed [SubLattice_isSubOrder of U by <: with disp] == [SubLattice_isSubOrder of U by <: ] == [SubPOrder_isSubOrder of U by <: with disp] == [SubPOrder_isSubOrder of U by <: ] == [SubChoice_isSubOrder of U by <: with disp] == [SubChoice_isSubOrder of U by <: ] == orderType mixin for a subType whose base type is an orderType [POrder of U by <: ] == porderType mixin for a subType whose base type is a porderType [Order of U by <: ] == orderType mixin for a subType whose base type is an orderType We provide expected instances of ordered types for bool, nat (for leq and and dvdn), 'I_n, 'I_n.+1 (with a top and bottom), nat for dvdn, T *prod[disp] T', T *lexi[disp] T', {t : T & T' x} (with lexicographic ordering), seqprod_with d T (using product order), seqlexi_with d T (with lexicographic ordering), n.-tupleprod[disp] (using product order), n.-tuplelexi[d] T (with lexicographic ordering), on {subset[disp] T} (using subset order) and all possible finite type instances. (Use `HB.about type` to discover the instances on type.) In order to get a canonical order on prod, seq, tuple or set, one may import modules DefaultProdOrder or DefaultProdLexiOrder, DefaultSeqProdOrder or DefaultSeqLexiOrder, DefaultTupleProdOrder or DefaultTupleLexiOrder, and DefaultSetSubsetOrder. We also provide specialized versions of some theorems from path.v. We provide Order.enum_val, Order.enum_rank, and Order.enum_rank_in, which are monotonous variations of enum_val, enum_rank, and enum_rank_in whenever the type is porderType, and their monotonicity is provided if this order is total. The theory is in the module Order (Order.enum_valK, Order.enum_rank_inK, etc) but Order.Enum can be imported to shorten these. We provide an opaque monotonous bijection tagnat.sig / tagnat.rank between the finite types {i : 'I_n & 'I_(p_ i)} and 'I_(\sum_i p_ i): tagnat.sig : 'I_(\sum_i p_ i) -> {i : 'I_n & 'I_(p_ i)} tagnat.rank : {i : 'I_n & 'I_(p_ i)} -> 'I_(\sum_i p_ i) tagnat.sig1 : 'I_(\sum_i p_ i) -> 'I_n tagnat.sig2 : forall p : 'I_(\sum_i p_ i), 'I_(p_ (tagnat.sig1 p)) tagnat.Rank : forall i, 'I_(p_ i) -> 'I_(\sum_i p_ i) Acknowledgments: This file is based on prior work by D. Dreyer, G. Gonthier, A. Nanevski, P-Y Strub, B. Ziliani

Set Implicit Arguments.

Declare Scope order_scope.

Delimit Scope order_scope with O.
Local Open Scope order_scope.

Reserved Notation "<= y" (at level 35).
Reserved Notation ">= y" (at level 35).
Reserved Notation "< y" (at level 35).
Reserved Notation "> y" (at level 35).
Reserved Notation "<= y :> T" (at level 35, y at next level).
Reserved Notation ">= y :> T" (at level 35, y at next level).
Reserved Notation "< y :> T" (at level 35, y at next level).
Reserved Notation "> y :> T" (at level 35, y at next level).
Reserved Notation "x >=< y" (at level 70, no associativity).
Reserved Notation ">=< y" (at level 35).
Reserved Notation ">=< y :> T" (at level 35, y at next level).
Reserved Notation "x >< y" (at level 70, no associativity).
Reserved Notation ">< x" (at level 35).
Reserved Notation ">< y :> T" (at level 35, y at next level).
Reserved Notation "f \min g" (at level 50, left associativity).
Reserved Notation "f \max g" (at level 50, left associativity).

Reserved Notation "x < y ?<= 'if' c" (at level 70, y, c at next level,
  format "x '[hv' < y '/' ?<= 'if' c ']'").
Reserved Notation "x < y ?<= 'if' c :> T" (at level 70, y, c at next level,
  format "x '[hv' < y '/' ?<= 'if' c :> T ']'").

Reserved notation for lattice operations.
Reserved Notation "A `&` B" (at level 48, left associativity).
Reserved Notation "A `|` B" (at level 52, left associativity).
Reserved Notation "A `\` B" (at level 50, left associativity).
Reserved Notation "~` A" (at level 35, right associativity).

Reserved notation for lattices with bottom/top elements.
Reserved Notation "0%O" (at level 0). (* deprecated in 1.17.0 *)
Reserved Notation "1%O" (at level 0). (* deprecated in 1.17.0 *)
Reserved Notation "\bot" (at level 0).
Reserved Notation "\top" (at level 0).

Notations for dual partial and total order
Reserved Notation "x <=^d y" (at level 70, y at next level).
Reserved Notation "x >=^d y" (at level 70, y at next level).
Reserved Notation "x <^d y" (at level 70, y at next level).
Reserved Notation "x >^d y" (at level 70, y at next level).
Reserved Notation "x <=^d y :> T" (at level 70, y at next level).
Reserved Notation "x >=^d y :> T" (at level 70, y at next level).
Reserved Notation "x <^d y :> T" (at level 70, y at next level).
Reserved Notation "x >^d y :> T" (at level 70, y at next level).
Reserved Notation "<=^d y" (at level 35).
Reserved Notation ">=^d y" (at level 35).
Reserved Notation "<^d y" (at level 35).
Reserved Notation ">^d y" (at level 35).
Reserved Notation "<=^d y :> T" (at level 35, y at next level).
Reserved Notation ">=^d y :> T" (at level 35, y at next level).
Reserved Notation "<^d y :> T" (at level 35, y at next level).
Reserved Notation ">^d y :> T" (at level 35, y at next level).
Reserved Notation "x >=<^d y" (at level 70, no associativity).
Reserved Notation ">=<^d y" (at level 35).
Reserved Notation ">=<^d y :> T" (at level 35, y at next level).
Reserved Notation "x ><^d y" (at level 70, no associativity).
Reserved Notation "><^d x" (at level 35).
Reserved Notation "><^d y :> T" (at level 35, y at next level).

Reserved Notation "x <=^d y <=^d z" (at level 70, y, z at next level).
Reserved Notation "x <^d y <=^d z" (at level 70, y, z at next level).
Reserved Notation "x <=^d y <^d z" (at level 70, y, z at next level).
Reserved Notation "x <^d y <^d z" (at level 70, y, z at next level).
Reserved Notation "x <=^d y ?= 'iff' c" (at level 70, y, c at next level,
  format "x '[hv' <=^d y '/' ?= 'iff' c ']'").
Reserved Notation "x <=^d y ?= 'iff' c :> T" (at level 70, y, c at next level,
  format "x '[hv' <=^d y '/' ?= 'iff' c :> T ']'").
Reserved Notation "x <^d y ?<= 'if' c" (at level 70, y, c at next level,
  format "x '[hv' <^d y '/' ?<= 'if' c ']'").
Reserved Notation "x <^d y ?<= 'if' c :> T" (at level 70, y, c at next level,
  format "x '[hv' <^d y '/' ?<= 'if' c :> T ']'").

Reserved notation for dual lattice operations.
Reserved Notation "A `&^d` B" (at level 48, left associativity).
Reserved Notation "A `|^d` B" (at level 52, left associativity).
Reserved Notation "A `\^d` B" (at level 50, left associativity).
Reserved Notation "~^d` A" (at level 35, right associativity).

Reserved Notation "0^d%O" (at level 0). (* deprecated in 1.17.0 *)
Reserved Notation "1^d%O" (at level 0). (* deprecated in 1.17.0 *)
Reserved Notation "\bot^d" (at level 0).
Reserved Notation "\top^d" (at level 0).

Reserved notations for product ordering of prod or seq
Reserved Notation "x <=^p y" (at level 70, y at next level).
Reserved Notation "x >=^p y" (at level 70, y at next level).
Reserved Notation "x <^p y" (at level 70, y at next level).
Reserved Notation "x >^p y" (at level 70, y at next level).
Reserved Notation "x <=^p y :> T" (at level 70, y at next level).
Reserved Notation "x >=^p y :> T" (at level 70, y at next level).
Reserved Notation "x <^p y :> T" (at level 70, y at next level).
Reserved Notation "x >^p y :> T" (at level 70, y at next level).
Reserved Notation "<=^p y" (at level 35).
Reserved Notation ">=^p y" (at level 35).
Reserved Notation "<^p y" (at level 35).
Reserved Notation ">^p y" (at level 35).
Reserved Notation "<=^p y :> T" (at level 35, y at next level).
Reserved Notation ">=^p y :> T" (at level 35, y at next level).
Reserved Notation "<^p y :> T" (at level 35, y at next level).
Reserved Notation ">^p y :> T" (at level 35, y at next level).
Reserved Notation "x >=<^p y" (at level 70, no associativity).
Reserved Notation ">=<^p x" (at level 35).
Reserved Notation ">=<^p y :> T" (at level 35, y at next level).
Reserved Notation "x ><^p y" (at level 70, no associativity).
Reserved Notation "><^p x" (at level 35).
Reserved Notation "><^p y :> T" (at level 35, y at next level).

Reserved Notation "x <=^p y <=^p z" (at level 70, y, z at next level).
Reserved Notation "x <^p y <=^p z" (at level 70, y, z at next level).
Reserved Notation "x <=^p y <^p z" (at level 70, y, z at next level).
Reserved Notation "x <^p y <^p z" (at level 70, y, z at next level).
Reserved Notation "x <=^p y ?= 'iff' c" (at level 70, y, c at next level,
  format "x '[hv' <=^p y '/' ?= 'iff' c ']'").
Reserved Notation "x <=^p y ?= 'iff' c :> T" (at level 70, y, c at next level,
  format "x '[hv' <=^p y '/' ?= 'iff' c :> T ']'").

Reserved notation for dual lattice operations.
Reserved Notation "A `&^p` B" (at level 48, left associativity).
Reserved Notation "A `|^p` B" (at level 52, left associativity).
Reserved Notation "A `\^p` B" (at level 50, left associativity).
Reserved Notation "~^p` A" (at level 35, right associativity).

Reserved notations for lexicographic ordering of prod or seq
Reserved Notation "x <=^l y" (at level 70, y at next level).
Reserved Notation "x >=^l y" (at level 70, y at next level).
Reserved Notation "x <^l y" (at level 70, y at next level).
Reserved Notation "x >^l y" (at level 70, y at next level).
Reserved Notation "x <=^l y :> T" (at level 70, y at next level).
Reserved Notation "x >=^l y :> T" (at level 70, y at next level).
Reserved Notation "x <^l y :> T" (at level 70, y at next level).
Reserved Notation "x >^l y :> T" (at level 70, y at next level).
Reserved Notation "<=^l y" (at level 35).
Reserved Notation ">=^l y" (at level 35).
Reserved Notation "<^l y" (at level 35).
Reserved Notation ">^l y" (at level 35).
Reserved Notation "<=^l y :> T" (at level 35, y at next level).
Reserved Notation ">=^l y :> T" (at level 35, y at next level).
Reserved Notation "<^l y :> T" (at level 35, y at next level).
Reserved Notation ">^l y :> T" (at level 35, y at next level).
Reserved Notation "x >=<^l y" (at level 70, no associativity).
Reserved Notation ">=<^l x" (at level 35).
Reserved Notation ">=<^l y :> T" (at level 35, y at next level).
Reserved Notation "x ><^l y" (at level 70, no associativity).
Reserved Notation "><^l x" (at level 35).
Reserved Notation "><^l y :> T" (at level 35, y at next level).

Reserved Notation "x <=^l y <=^l z" (at level 70, y, z at next level).
Reserved Notation "x <^l y <=^l z" (at level 70, y, z at next level).
Reserved Notation "x <=^l y <^l z" (at level 70, y, z at next level).
Reserved Notation "x <^l y <^l z" (at level 70, y, z at next level).
Reserved Notation "x <=^l y ?= 'iff' c" (at level 70, y, c at next level,
  format "x '[hv' <=^l y '/' ?= 'iff' c ']'").
Reserved Notation "x <=^l y ?= 'iff' c :> T" (at level 70, y, c at next level,
  format "x '[hv' <=^l y '/' ?= 'iff' c :> T ']'").

Reserved notations for divisibility
Reserved Notation "x %<| y" (at level 70, no associativity).

Reserved Notation "\gcd_ i F"
  (at level 41, F at level 41, i at level 0,
           format "'[' \gcd_ i '/ ' F ']'").
Reserved Notation "\gcd_ ( i <- r | P ) F"
  (at level 41, F at level 41, i, r at level 50,
           format "'[' \gcd_ ( i <- r | P ) '/ ' F ']'").
Reserved Notation "\gcd_ ( i <- r ) F"
  (at level 41, F at level 41, i, r at level 50,
           format "'[' \gcd_ ( i <- r ) '/ ' F ']'").
Reserved Notation "\gcd_ ( m <= i < n | P ) F"
  (at level 41, F at level 41, i, m, n at level 50,
           format "'[' \gcd_ ( m <= i < n | P ) '/ ' F ']'").
Reserved Notation "\gcd_ ( m <= i < n ) F"
  (at level 41, F at level 41, i, m, n at level 50,
           format "'[' \gcd_ ( m <= i < n ) '/ ' F ']'").
Reserved Notation "\gcd_ ( i | P ) F"
  (at level 41, F at level 41, i at level 50,
           format "'[' \gcd_ ( i | P ) '/ ' F ']'").
Reserved Notation "\gcd_ ( i : t | P ) F"
  (at level 41, F at level 41, i at level 50).
Reserved Notation "\gcd_ ( i : t ) F"
  (at level 41, F at level 41, i at level 50).
Reserved Notation "\gcd_ ( i < n | P ) F"
  (at level 41, F at level 41, i, n at level 50,
           format "'[' \gcd_ ( i < n | P ) '/ ' F ']'").
Reserved Notation "\gcd_ ( i < n ) F"
  (at level 41, F at level 41, i, n at level 50,
           format "'[' \gcd_ ( i < n ) F ']'").
Reserved Notation "\gcd_ ( i 'in' A | P ) F"
  (at level 41, F at level 41, i, A at level 50,
           format "'[' \gcd_ ( i 'in' A | P ) '/ ' F ']'").
Reserved Notation "\gcd_ ( i 'in' A ) F"
  (at level 41, F at level 41, i, A at level 50,
           format "'[' \gcd_ ( i 'in' A ) '/ ' F ']'").

Reserved Notation "\lcm_ i F"
  (at level 41, F at level 41, i at level 0,
           format "'[' \lcm_ i '/ ' F ']'").
Reserved Notation "\lcm_ ( i <- r | P ) F"
  (at level 41, F at level 41, i, r at level 50,
           format "'[' \lcm_ ( i <- r | P ) '/ ' F ']'").
Reserved Notation "\lcm_ ( i <- r ) F"
  (at level 41, F at level 41, i, r at level 50,
           format "'[' \lcm_ ( i <- r ) '/ ' F ']'").
Reserved Notation "\lcm_ ( m <= i < n | P ) F"
  (at level 41, F at level 41, i, m, n at level 50,
           format "'[' \lcm_ ( m <= i < n | P ) '/ ' F ']'").
Reserved Notation "\lcm_ ( m <= i < n ) F"
  (at level 41, F at level 41, i, m, n at level 50,
           format "'[' \lcm_ ( m <= i < n ) '/ ' F ']'").
Reserved Notation "\lcm_ ( i | P ) F"
  (at level 41, F at level 41, i at level 50,
           format "'[' \lcm_ ( i | P ) '/ ' F ']'").
Reserved Notation "\lcm_ ( i : t | P ) F"
  (at level 41, F at level 41, i at level 50).
Reserved Notation "\lcm_ ( i : t ) F"
  (at level 41, F at level 41, i at level 50).
Reserved Notation "\lcm_ ( i < n | P ) F"
  (at level 41, F at level 41, i, n at level 50,
           format "'[' \lcm_ ( i < n | P ) '/ ' F ']'").
Reserved Notation "\lcm_ ( i < n ) F"
  (at level 41, F at level 41, i, n at level 50,
           format "'[' \lcm_ ( i < n ) F ']'").
Reserved Notation "\lcm_ ( i 'in' A | P ) F"
  (at level 41, F at level 41, i, A at level 50,
           format "'[' \lcm_ ( i 'in' A | P ) '/ ' F ']'").
Reserved Notation "\lcm_ ( i 'in' A ) F"
  (at level 41, F at level 41, i, A at level 50,
           format "'[' \lcm_ ( i 'in' A ) '/ ' F ']'").

Reserved notation for dual lattice operations.
Reserved Notation "A `&^l` B" (at level 48, left associativity).
Reserved Notation "A `|^l` B" (at level 52, left associativity).
Reserved Notation "A `\^l` B" (at level 50, left associativity).
Reserved Notation "~^l` A" (at level 35, right associativity).

Reserved Notation "\meet_ i F"
  (at level 41, F at level 41, i at level 0,
           format "'[' \meet_ i '/ ' F ']'").
Reserved Notation "\meet_ ( i <- r | P ) F"
  (at level 41, F at level 41, i, r at level 50,
           format "'[' \meet_ ( i <- r | P ) '/ ' F ']'").
Reserved Notation "\meet_ ( i <- r ) F"
  (at level 41, F at level 41, i, r at level 50,
           format "'[' \meet_ ( i <- r ) '/ ' F ']'").
Reserved Notation "\meet_ ( m <= i < n | P ) F"
  (at level 41, F at level 41, i, m, n at level 50,
           format "'[' \meet_ ( m <= i < n | P ) '/ ' F ']'").
Reserved Notation "\meet_ ( m <= i < n ) F"
  (at level 41, F at level 41, i, m, n at level 50,
           format "'[' \meet_ ( m <= i < n ) '/ ' F ']'").
Reserved Notation "\meet_ ( i | P ) F"
  (at level 41, F at level 41, i at level 50,
           format "'[' \meet_ ( i | P ) '/ ' F ']'").
Reserved Notation "\meet_ ( i : t | P ) F"
  (at level 41, F at level 41, i at level 50).
Reserved Notation "\meet_ ( i : t ) F"
  (at level 41, F at level 41, i at level 50).
Reserved Notation "\meet_ ( i < n | P ) F"
  (at level 41, F at level 41, i, n at level 50,
           format "'[' \meet_ ( i < n | P ) '/ ' F ']'").
Reserved Notation "\meet_ ( i < n ) F"
  (at level 41, F at level 41, i, n at level 50,
           format "'[' \meet_ ( i < n ) F ']'").
Reserved Notation "\meet_ ( i 'in' A | P ) F"
  (at level 41, F at level 41, i, A at level 50,
           format "'[' \meet_ ( i 'in' A | P ) '/ ' F ']'").
Reserved Notation "\meet_ ( i 'in' A ) F"
  (at level 41, F at level 41, i, A at level 50,
           format "'[' \meet_ ( i 'in' A ) '/ ' F ']'").

Reserved Notation "\join_ i F"
  (at level 41, F at level 41, i at level 0,
           format "'[' \join_ i '/ ' F ']'").
Reserved Notation "\join_ ( i <- r | P ) F"
  (at level 41, F at level 41, i, r at level 50,
           format "'[' \join_ ( i <- r | P ) '/ ' F ']'").
Reserved Notation "\join_ ( i <- r ) F"
  (at level 41, F at level 41, i, r at level 50,
           format "'[' \join_ ( i <- r ) '/ ' F ']'").
Reserved Notation "\join_ ( m <= i < n | P ) F"
  (at level 41, F at level 41, i, m, n at level 50,
           format "'[' \join_ ( m <= i < n | P ) '/ ' F ']'").
Reserved Notation "\join_ ( m <= i < n ) F"
  (at level 41, F at level 41, i, m, n at level 50,
           format "'[' \join_ ( m <= i < n ) '/ ' F ']'").
Reserved Notation "\join_ ( i | P ) F"
  (at level 41, F at level 41, i at level 50,
           format "'[' \join_ ( i | P ) '/ ' F ']'").
Reserved Notation "\join_ ( i : t | P ) F"
  (at level 41, F at level 41, i at level 50).
Reserved Notation "\join_ ( i : t ) F"
  (at level 41, F at level 41, i at level 50).
Reserved Notation "\join_ ( i < n | P ) F"
  (at level 41, F at level 41, i, n at level 50,
           format "'[' \join_ ( i < n | P ) '/ ' F ']'").
Reserved Notation "\join_ ( i < n ) F"
  (at level 41, F at level 41, i, n at level 50,
           format "'[' \join_ ( i < n ) F ']'").
Reserved Notation "\join_ ( i 'in' A | P ) F"
  (at level 41, F at level 41, i, A at level 50,
           format "'[' \join_ ( i 'in' A | P ) '/ ' F ']'").
Reserved Notation "\join_ ( i 'in' A ) F"
  (at level 41, F at level 41, i, A at level 50,
           format "'[' \join_ ( i 'in' A ) '/ ' F ']'").

Reserved Notation "\min_ i F"
  (at level 41, F at level 41, i at level 0,
           format "'[' \min_ i '/ ' F ']'").
Reserved Notation "\min_ ( i <- r | P ) F"
  (at level 41, F at level 41, i, r at level 50,
           format "'[' \min_ ( i <- r | P ) '/ ' F ']'").
Reserved Notation "\min_ ( i <- r ) F"
  (at level 41, F at level 41, i, r at level 50,
           format "'[' \min_ ( i <- r ) '/ ' F ']'").
Reserved Notation "\min_ ( m <= i < n | P ) F"
  (at level 41, F at level 41, i, m, n at level 50,
           format "'[' \min_ ( m <= i < n | P ) '/ ' F ']'").
Reserved Notation "\min_ ( m <= i < n ) F"
  (at level 41, F at level 41, i, m, n at level 50,
           format "'[' \min_ ( m <= i < n ) '/ ' F ']'").
Reserved Notation "\min_ ( i | P ) F"
  (at level 41, F at level 41, i at level 50,
           format "'[' \min_ ( i | P ) '/ ' F ']'").
Reserved Notation "\min_ ( i : t | P ) F"
  (at level 41, F at level 41, i at level 50).
Reserved Notation "\min_ ( i : t ) F"
  (at level 41, F at level 41, i at level 50).
Reserved Notation "\min_ ( i < n | P ) F"
  (at level 41, F at level 41, i, n at level 50,
           format "'[' \min_ ( i < n | P ) '/ ' F ']'").
Reserved Notation "\min_ ( i < n ) F"
  (at level 41, F at level 41, i, n at level 50,
           format "'[' \min_ ( i < n ) F ']'").
Reserved Notation "\min_ ( i 'in' A | P ) F"
  (at level 41, F at level 41, i, A at level 50,
           format "'[' \min_ ( i 'in' A | P ) '/ ' F ']'").
Reserved Notation "\min_ ( i 'in' A ) F"
  (at level 41, F at level 41, i, A at level 50,
           format "'[' \min_ ( i 'in' A ) '/ ' F ']'").

Reserved Notation "\max_ i F"
  (at level 41, F at level 41, i at level 0,
           format "'[' \max_ i '/ ' F ']'").
Reserved Notation "\max_ ( i <- r | P ) F"
  (at level 41, F at level 41, i, r at level 50,
           format "'[' \max_ ( i <- r | P ) '/ ' F ']'").
Reserved Notation "\max_ ( i <- r ) F"
  (at level 41, F at level 41, i, r at level 50,
           format "'[' \max_ ( i <- r ) '/ ' F ']'").
Reserved Notation "\max_ ( m <= i < n | P ) F"
  (at level 41, F at level 41, i, m, n at level 50,
           format "'[' \max_ ( m <= i < n | P ) '/ ' F ']'").
Reserved Notation "\max_ ( m <= i < n ) F"
  (at level 41, F at level 41, i, m, n at level 50,
           format "'[' \max_ ( m <= i < n ) '/ ' F ']'").
Reserved Notation "\max_ ( i | P ) F"
  (at level 41, F at level 41, i at level 50,
           format "'[' \max_ ( i | P ) '/ ' F ']'").
Reserved Notation "\max_ ( i : t | P ) F"
  (at level 41, F at level 41, i at level 50).
Reserved Notation "\max_ ( i : t ) F"
  (at level 41, F at level 41, i at level 50).
Reserved Notation "\max_ ( i < n | P ) F"
  (at level 41, F at level 41, i, n at level 50,
           format "'[' \max_ ( i < n | P ) '/ ' F ']'").
Reserved Notation "\max_ ( i < n ) F"
  (at level 41, F at level 41, i, n at level 50,
           format "'[' \max_ ( i < n ) F ']'").
Reserved Notation "\max_ ( i 'in' A | P ) F"
  (at level 41, F at level 41, i, A at level 50,
           format "'[' \max_ ( i 'in' A | P ) '/ ' F ']'").
Reserved Notation "\max_ ( i 'in' A ) F"
  (at level 41, F at level 41, i, A at level 50,
           format "'[' \max_ ( i 'in' A ) '/ ' F ']'").

Reserved Notation "\meet^d_ i F"
  (at level 41, F at level 41, i at level 0,
           format "'[' \meet^d_ i '/ ' F ']'").
Reserved Notation "\meet^d_ ( i <- r | P ) F"
  (at level 41, F at level 41, i, r at level 50,
           format "'[' \meet^d_ ( i <- r | P ) '/ ' F ']'").
Reserved Notation "\meet^d_ ( i <- r ) F"
  (at level 41, F at level 41, i, r at level 50,
           format "'[' \meet^d_ ( i <- r ) '/ ' F ']'").
Reserved Notation "\meet^d_ ( m <= i < n | P ) F"
  (at level 41, F at level 41, i, m, n at level 50,
           format "'[' \meet^d_ ( m <= i < n | P ) '/ ' F ']'").
Reserved Notation "\meet^d_ ( m <= i < n ) F"
  (at level 41, F at level 41, i, m, n at level 50,
           format "'[' \meet^d_ ( m <= i < n ) '/ ' F ']'").
Reserved Notation "\meet^d_ ( i | P ) F"
  (at level 41, F at level 41, i at level 50,
           format "'[' \meet^d_ ( i | P ) '/ ' F ']'").
Reserved Notation "\meet^d_ ( i : t | P ) F"
  (at level 41, F at level 41, i at level 50).
Reserved Notation "\meet^d_ ( i : t ) F"
  (at level 41, F at level 41, i at level 50).
Reserved Notation "\meet^d_ ( i < n | P ) F"
  (at level 41, F at level 41, i, n at level 50,
           format "'[' \meet^d_ ( i < n | P ) '/ ' F ']'").
Reserved Notation "\meet^d_ ( i < n ) F"
  (at level 41, F at level 41, i, n at level 50,
           format "'[' \meet^d_ ( i < n ) F ']'").
Reserved Notation "\meet^d_ ( i 'in' A | P ) F"
  (at level 41, F at level 41, i, A at level 50,
           format "'[' \meet^d_ ( i 'in' A | P ) '/ ' F ']'").
Reserved Notation "\meet^d_ ( i 'in' A ) F"
  (at level 41, F at level 41, i, A at level 50,
           format "'[' \meet^d_ ( i 'in' A ) '/ ' F ']'").

Reserved Notation "\join^d_ i F"
  (at level 41, F at level 41, i at level 0,
           format "'[' \join^d_ i '/ ' F ']'").
Reserved Notation "\join^d_ ( i <- r | P ) F"
  (at level 41, F at level 41, i, r at level 50,
           format "'[' \join^d_ ( i <- r | P ) '/ ' F ']'").
Reserved Notation "\join^d_ ( i <- r ) F"
  (at level 41, F at level 41, i, r at level 50,
           format "'[' \join^d_ ( i <- r ) '/ ' F ']'").
Reserved Notation "\join^d_ ( m <= i < n | P ) F"
  (at level 41, F at level 41, i, m, n at level 50,
           format "'[' \join^d_ ( m <= i < n | P ) '/ ' F ']'").
Reserved Notation "\join^d_ ( m <= i < n ) F"
  (at level 41, F at level 41, i, m, n at level 50,
           format "'[' \join^d_ ( m <= i < n ) '/ ' F ']'").
Reserved Notation "\join^d_ ( i | P ) F"
  (at level 41, F at level 41, i at level 50,
           format "'[' \join^d_ ( i | P ) '/ ' F ']'").
Reserved Notation "\join^d_ ( i : t | P ) F"
  (at level 41, F at level 41, i at level 50).
Reserved Notation "\join^d_ ( i : t ) F"
  (at level 41, F at level 41, i at level 50).
Reserved Notation "\join^d_ ( i < n | P ) F"
  (at level 41, F at level 41, i, n at level 50,
           format "'[' \join^d_ ( i < n | P ) '/ ' F ']'").
Reserved Notation "\join^d_ ( i < n ) F"
  (at level 41, F at level 41, i, n at level 50,
           format "'[' \join^d_ ( i < n ) F ']'").
Reserved Notation "\join^d_ ( i 'in' A | P ) F"
  (at level 41, F at level 41, i, A at level 50,
           format "'[' \join^d_ ( i 'in' A | P ) '/ ' F ']'").
Reserved Notation "\join^d_ ( i 'in' A ) F"
  (at level 41, F at level 41, i, A at level 50,
           format "'[' \join^d_ ( i 'in' A ) '/ ' F ']'").

Reserved Notation "\min^d_ i F"
  (at level 41, F at level 41, i at level 0,
           format "'[' \min^d_ i '/ ' F ']'").
Reserved Notation "\min^d_ ( i <- r | P ) F"
  (at level 41, F at level 41, i, r at level 50,
           format "'[' \min^d_ ( i <- r | P ) '/ ' F ']'").
Reserved Notation "\min^d_ ( i <- r ) F"
  (at level 41, F at level 41, i, r at level 50,
           format "'[' \min^d_ ( i <- r ) '/ ' F ']'").
Reserved Notation "\min^d_ ( m <= i < n | P ) F"
  (at level 41, F at level 41, i, m, n at level 50,
           format "'[' \min^d_ ( m <= i < n | P ) '/ ' F ']'").
Reserved Notation "\min^d_ ( m <= i < n ) F"
  (at level 41, F at level 41, i, m, n at level 50,
           format "'[' \min^d_ ( m <= i < n ) '/ ' F ']'").
Reserved Notation "\min^d_ ( i | P ) F"
  (at level 41, F at level 41, i at level 50,
           format "'[' \min^d_ ( i | P ) '/ ' F ']'").
Reserved Notation "\min^d_ ( i : t | P ) F"
  (at level 41, F at level 41, i at level 50).
Reserved Notation "\min^d_ ( i : t ) F"
  (at level 41, F at level 41, i at level 50).
Reserved Notation "\min^d_ ( i < n | P ) F"
  (at level 41, F at level 41, i, n at level 50,
           format "'[' \min^d_ ( i < n | P ) '/ ' F ']'").
Reserved Notation "\min^d_ ( i < n ) F"
  (at level 41, F at level 41, i, n at level 50,
           format "'[' \min^d_ ( i < n ) F ']'").
Reserved Notation "\min^d_ ( i 'in' A | P ) F"
  (at level 41, F at level 41, i, A at level 50,
           format "'[' \min^d_ ( i 'in' A | P ) '/ ' F ']'").
Reserved Notation "\min^d_ ( i 'in' A ) F"
  (at level 41, F at level 41, i, A at level 50,
           format "'[' \min^d_ ( i 'in' A ) '/ ' F ']'").

Reserved Notation "\max^d_ i F"
  (at level 41, F at level 41, i at level 0,
           format "'[' \max^d_ i '/ ' F ']'").
Reserved Notation "\max^d_ ( i <- r | P ) F"
  (at level 41, F at level 41, i, r at level 50,
           format "'[' \max^d_ ( i <- r | P ) '/ ' F ']'").
Reserved Notation "\max^d_ ( i <- r ) F"
  (at level 41, F at level 41, i, r at level 50,
           format "'[' \max^d_ ( i <- r ) '/ ' F ']'").
Reserved Notation "\max^d_ ( m <= i < n | P ) F"
  (at level 41, F at level 41, i, m, n at level 50,
           format "'[' \max^d_ ( m <= i < n | P ) '/ ' F ']'").
Reserved Notation "\max^d_ ( m <= i < n ) F"
  (at level 41, F at level 41, i, m, n at level 50,
           format "'[' \max^d_ ( m <= i < n ) '/ ' F ']'").
Reserved Notation "\max^d_ ( i | P ) F"
  (at level 41, F at level 41, i at level 50,
           format "'[' \max^d_ ( i | P ) '/ ' F ']'").
Reserved Notation "\max^d_ ( i : t | P ) F"
  (at level 41, F at level 41, i at level 50).
Reserved Notation "\max^d_ ( i : t ) F"
  (at level 41, F at level 41, i at level 50).
Reserved Notation "\max^d_ ( i < n | P ) F"
  (at level 41, F at level 41, i, n at level 50,
           format "'[' \max^d_ ( i < n | P ) '/ ' F ']'").
Reserved Notation "\max^d_ ( i < n ) F"
  (at level 41, F at level 41, i, n at level 50,
           format "'[' \max^d_ ( i < n ) F ']'").
Reserved Notation "\max^d_ ( i 'in' A | P ) F"
  (at level 41, F at level 41, i, A at level 50,
           format "'[' \max^d_ ( i 'in' A | P ) '/ ' F ']'").
Reserved Notation "\max^d_ ( i 'in' A ) F"
  (at level 41, F at level 41, i, A at level 50,
           format "'[' \max^d_ ( i 'in' A ) '/ ' F ']'").

Reserved Notation "\meet^p_ i F"
  (at level 41, F at level 41, i at level 0,
           format "'[' \meet^p_ i '/ ' F ']'").
Reserved Notation "\meet^p_ ( i <- r | P ) F"
  (at level 41, F at level 41, i, r at level 50,
           format "'[' \meet^p_ ( i <- r | P ) '/ ' F ']'").
Reserved Notation "\meet^p_ ( i <- r ) F"
  (at level 41, F at level 41, i, r at level 50,
           format "'[' \meet^p_ ( i <- r ) '/ ' F ']'").
Reserved Notation "\meet^p_ ( m <= i < n | P ) F"
  (at level 41, F at level 41, i, m, n at level 50,
           format "'[' \meet^p_ ( m <= i < n | P ) '/ ' F ']'").
Reserved Notation "\meet^p_ ( m <= i < n ) F"
  (at level 41, F at level 41, i, m, n at level 50,
           format "'[' \meet^p_ ( m <= i < n ) '/ ' F ']'").
Reserved Notation "\meet^p_ ( i | P ) F"
  (at level 41, F at level 41, i at level 50,
           format "'[' \meet^p_ ( i | P ) '/ ' F ']'").
Reserved Notation "\meet^p_ ( i : t | P ) F"
  (at level 41, F at level 41, i at level 50).
Reserved Notation "\meet^p_ ( i : t ) F"
  (at level 41, F at level 41, i at level 50).
Reserved Notation "\meet^p_ ( i < n | P ) F"
  (at level 41, F at level 41, i, n at level 50,
           format "'[' \meet^p_ ( i < n | P ) '/ ' F ']'").
Reserved Notation "\meet^p_ ( i < n ) F"
  (at level 41, F at level 41, i, n at level 50,
           format "'[' \meet^p_ ( i < n ) F ']'").
Reserved Notation "\meet^p_ ( i 'in' A | P ) F"
  (at level 41, F at level 41, i, A at level 50,
           format "'[' \meet^p_ ( i 'in' A | P ) '/ ' F ']'").
Reserved Notation "\meet^p_ ( i 'in' A ) F"
  (at level 41, F at level 41, i, A at level 50,
           format "'[' \meet^p_ ( i 'in' A ) '/ ' F ']'").

Reserved Notation "\join^p_ i F"
  (at level 41, F at level 41, i at level 0,
           format "'[' \join^p_ i '/ ' F ']'").
Reserved Notation "\join^p_ ( i <- r | P ) F"
  (at level 41, F at level 41, i, r at level 50,
           format "'[' \join^p_ ( i <- r | P ) '/ ' F ']'").
Reserved Notation "\join^p_ ( i <- r ) F"
  (at level 41, F at level 41, i, r at level 50,
           format "'[' \join^p_ ( i <- r ) '/ ' F ']'").
Reserved Notation "\join^p_ ( m <= i < n | P ) F"
  (at level 41, F at level 41, i, m, n at level 50,
           format "'[' \join^p_ ( m <= i < n | P ) '/ ' F ']'").
Reserved Notation "\join^p_ ( m <= i < n ) F"
  (at level 41, F at level 41, i, m, n at level 50,
           format "'[' \join^p_ ( m <= i < n ) '/ ' F ']'").
Reserved Notation "\join^p_ ( i | P ) F"
  (at level 41, F at level 41, i at level 50,
           format "'[' \join^p_ ( i | P ) '/ ' F ']'").
Reserved Notation "\join^p_ ( i : t | P ) F"
  (at level 41, F at level 41, i at level 50).
Reserved Notation "\join^p_ ( i : t ) F"
  (at level 41, F at level 41, i at level 50).
Reserved Notation "\join^p_ ( i < n | P ) F"
  (at level 41, F at level 41, i, n at level 50,
           format "'[' \join^p_ ( i < n | P ) '/ ' F ']'").
Reserved Notation "\join^p_ ( i < n ) F"
  (at level 41, F at level 41, i, n at level 50,
           format "'[' \join^p_ ( i < n ) F ']'").
Reserved Notation "\join^p_ ( i 'in' A | P ) F"
  (at level 41, F at level 41, i, A at level 50,
           format "'[' \join^p_ ( i 'in' A | P ) '/ ' F ']'").
Reserved Notation "\join^p_ ( i 'in' A ) F"
  (at level 41, F at level 41, i, A at level 50,
           format "'[' \join^p_ ( i 'in' A ) '/ ' F ']'").

Reserved Notation "'{' 'omorphism' U '->' V '}'"
  (at level 0, U at level 98, V at level 99,
   format "{ 'omorphism' U -> V }").
Reserved Notation "'{' 'mlmorphism' U '->' V '}'"
  (at level 0, U at level 98, V at level 99,
   format "{ 'mlmorphism' U -> V }").
Reserved Notation "'{' 'jlmorphism' U '->' V '}'"
  (at level 0, U at level 98, V at level 99,
   format "{ 'jlmorphism' U -> V }").
Reserved Notation "'{' 'lmorphism' U '->' V '}'"
  (at level 0, U at level 98, V at level 99,
   format "{ 'lmorphism' U -> V }").
Reserved Notation "'{' 'blmorphism' U '->' V '}'"
  (at level 0, U at level 98, V at level 99,
   format "{ 'blmorphism' U -> V }").
Reserved Notation "'{' 'tlmorphism' U '->' V '}'"
  (at level 0, U at level 98, V at level 99,
   format "{ 'tlmorphism' U -> V }").
Reserved Notation "'{' 'tblmorphism' U '->' V '}'"
  (at level 0, U at level 98, V at level 99,
   format "{ 'tblmorphism' U -> V }").

Module Order.


#[short(type="porderType")]
HB.structure Definition POrder (d : unit) :=
  { T of Choice T & isPOrder d T }.


TODO: print nice error message when keyed type is not provided


Let le_refl : reflexive le.

Let le_anti : antisymmetric le.

Let le_trans : transitive le.

Let lt_def x y : lt x y = (y != x) && (le x y).



#[key="T"]
HB.builders Context (d : unit) (T : Type) of Lt_isPOrder d T.

Module POrderExports.
Arguments le_trans {d s} [_ _ _].
#[deprecated(since="mathcomp 2.0.0", note="Use POrder.clone instead.")]
Notation "[ 'porderType' 'of' T 'for' cT ]" := (POrder.clone _ T%type cT)
  (at level 0, format "[ 'porderType' 'of' T 'for' cT ]") : form_scope.
#[deprecated(since="mathcomp 2.0.0", note="Use POrder.clone instead.")]
Notation "[ 'porderType' 'of' T 'for' cT 'with' disp ]" :=
  (POrder.clone disp T%type cT)
  (at level 0, format "[ 'porderType' 'of' T 'for' cT 'with' disp ]") :
  form_scope.
#[deprecated(since="mathcomp 2.0.0", note="Use POrder.clone instead.")]
Notation "[ 'porderType' 'of' T ]" := (POrder.clone _ T%type _)
  (at level 0, format "[ 'porderType' 'of' T ]") : form_scope.
#[deprecated(since="mathcomp 2.0.0", note="Use POrder.clone instead.")]
Notation "[ 'porderType' 'of' T 'with' disp ]" := (POrder.clone disp T%type _)
  (at level 0, format "[ 'porderType' 'of' T 'with' disp ]") : form_scope.
End POrderExports.
Bind Scope order_scope with POrder.sort.

Section POrderDef.

Variable (disp : unit) (T : porderType disp).


Definition comparable : rel T := fun (x y : T) ⇒ (x y) || (y x).

Definition ge : simpl_rel T := [rel x y | y x].
Definition gt : simpl_rel T := [rel x y | y < x].
Definition leif (x y : T) C : Prop := ((x y) × ((x == y) = C))%type.

Definition le_of_leif x y C (le_xy : @leif x y C) := le_xy.1 : le x y.

Definition lteif (x y : T) C := if C then x y else x < y.

Variant le_xor_gt (x y : T) :
  T T T T bool bool Set :=
  | LeNotGt of x y : le_xor_gt x y x x y y true false
  | GtNotLe of y < x : le_xor_gt x y y y x x false true.

Variant lt_xor_ge (x y : T) :
  T T T T bool bool Set :=
  | LtNotGe of x < y : lt_xor_ge x y x x y y false true
  | GeNotLt of y x : lt_xor_ge x y y y x x true false.

Definition min (x y : T) := if x < y then x else y.
Definition max (x y : T) := if x < y then y else x.

Variant compare (x y : T) :
   T T T T
   bool bool bool bool bool bool Set :=
  | CompareLt of x < y : compare x y
    x x y y false false false true false true
  | CompareGt of y < x : compare x y
    y y x x false false true false true false
  | CompareEq of x = y : compare x y
    x x x x true true true true false false.

Variant incompare (x y : T) :
   T T T T
  bool bool bool bool bool bool bool bool Set :=
  | InCompareLt of x < y : incompare x y
    x x y y false false false true false true true true
  | InCompareGt of y < x : incompare x y
    y y x x false false true false true false true true
  | InCompare of x >< y : incompare x y
    x y y x false false false false false false false false
  | InCompareEq of x = y : incompare x y
    x x x x true true true true false false true true.

Definition arg_min {I : finType} := @extremum T I le.
Definition arg_max {I : finType} := @extremum T I ge.

Lifted min/max operations.
Section LiftedPOrder.
Variable T' : Type.
Implicit Type f : T' T.
Definition min_fun f g x := min (f x) (g x).
Definition max_fun f g x := max (f x) (g x).
End LiftedPOrder.

End POrderDef.

Arguments ge {_ _}.
Arguments gt {_ _}.
Arguments min {_ _}.
Arguments max {_ _}.
Arguments comparable {_ _}.
Arguments min_fun {_ _ _} f g _ /.
Arguments max_fun {_ _ _} f g _ /.

Module Import POSyntax.

Notation "<=%O" := le : function_scope.
Notation ">=%O" := ge : function_scope.
Notation "<%O" := lt : function_scope.
Notation ">%O" := gt : function_scope.
Notation "<?=%O" := leif : function_scope.
Notation "<?<=%O" := lteif : function_scope.
Notation ">=<%O" := comparable : function_scope.
Notation "><%O" := (fun x y~~ (comparable x y)) : function_scope.

Notation "<= y" := (ge y) : order_scope.
Notation "<= y :> T" := ( (y : T)) (only parsing) : order_scope.
Notation ">= y" := (le y) : order_scope.
Notation ">= y :> T" := ( (y : T)) (only parsing) : order_scope.

Notation "< y" := (gt y) : order_scope.
Notation "< y :> T" := (< (y : T)) (only parsing) : order_scope.
Notation "> y" := (lt y) : order_scope.
Notation "> y :> T" := (> (y : T)) (only parsing) : order_scope.

Notation "x <= y" := (le x y) : order_scope.
Notation "x <= y :> T" := ((x : T) (y : T)) (only parsing) : order_scope.
Notation "x >= y" := (y x) (only parsing) : order_scope.
Notation "x >= y :> T" := ((x : T) (y : T)) (only parsing) : order_scope.

Notation "x < y" := (lt x y) : order_scope.
Notation "x < y :> T" := ((x : T) < (y : T)) (only parsing) : order_scope.
Notation "x > y" := (y < x) (only parsing) : order_scope.
Notation "x > y :> T" := ((x : T) > (y : T)) (only parsing) : order_scope.

Notation "x <= y <= z" := ((x y) && (y z)) : order_scope.
Notation "x < y <= z" := ((x < y) && (y z)) : order_scope.
Notation "x <= y < z" := ((x y) && (y < z)) : order_scope.
Notation "x < y < z" := ((x < y) && (y < z)) : order_scope.

Notation "x <= y ?= 'iff' C" := (leif x y C) : order_scope.
Notation "x <= y ?= 'iff' C :> T" := ((x : T) (y : T) ?= iff C)
  (only parsing) : order_scope.

Notation "x < y ?<= 'if' C" := (lteif x y C) : order_scope.
Notation "x < y ?<= 'if' C :> T" := ((x : T) < (y : T) ?<= if C)
  (only parsing) : order_scope.

Notation ">=< y" := [pred x | comparable x y] : order_scope.
Notation ">=< y :> T" := (>=< (y : T)) (only parsing) : order_scope.
Notation "x >=< y" := (comparable x y) : order_scope.

Notation ">< y" := [pred x | ~~ comparable x y] : order_scope.
Notation ">< y :> T" := (>< (y : T)) (only parsing) : order_scope.
Notation "x >< y" := (~~ (comparable x y)) : order_scope.

Notation "[ 'arg' 'min_' ( i < i0 | P ) F ]" :=
    (arg_min i0 (fun iP%B) (fun iF))
  (at level 0, i, i0 at level 10,
   format "[ 'arg' 'min_' ( i < i0 | P ) F ]") : order_scope.

Notation "[ 'arg' 'min_' ( i < i0 'in' A ) F ]" :=
    [arg min_(i < i0 | i \in A) F]
  (at level 0, i, i0 at level 10,
   format "[ 'arg' 'min_' ( i < i0 'in' A ) F ]") : order_scope.

Notation "[ 'arg' 'min_' ( i < i0 ) F ]" := [arg min_(i < i0 | true) F]
  (at level 0, i, i0 at level 10,
   format "[ 'arg' 'min_' ( i < i0 ) F ]") : order_scope.

Notation "[ 'arg' 'max_' ( i > i0 | P ) F ]" :=
     (arg_max i0 (fun iP%B) (fun iF))
  (at level 0, i, i0 at level 10,
   format "[ 'arg' 'max_' ( i > i0 | P ) F ]") : order_scope.

Notation "[ 'arg' 'max_' ( i > i0 'in' A ) F ]" :=
    [arg max_(i > i0 | i \in A) F]
  (at level 0, i, i0 at level 10,
   format "[ 'arg' 'max_' ( i > i0 'in' A ) F ]") : order_scope.

Notation "[ 'arg' 'max_' ( i > i0 ) F ]" := [arg max_(i > i0 | true) F]
  (at level 0, i, i0 at level 10,
   format "[ 'arg' 'max_' ( i > i0 ) F ]") : order_scope.

Notation "f \min g" := (min_fun f g) : function_scope.
Notation "f \max g" := (max_fun f g) : function_scope.

Notation leLHS := (X in (X _)%O)%pattern.
Notation leRHS := (X in (_ X)%O)%pattern.
Notation ltLHS := (X in (X < _)%O)%pattern.
Notation ltRHS := (X in (_ < X)%O)%pattern.

End POSyntax.

Module POCoercions.
Coercion le_of_leif : leif >-> is_true.
End POCoercions.

HB.mixin Record POrder_isJoinSemiLattice d (T : indexed Type) of POrder d T := { join : T -> T -> T; joinC : commutative join; joinA : associative join; le_defU : forall x y, (x <= y) = (join x y == y); }. # [short(type="joinSemiLatticeType") ] HB.structure Definition JoinSemiLattice d := { T of POrder_isJoinSemiLattice d T & POrder d T }. HB.mixin Record POrder_isMeetSemiLattice d (T : indexed Type) of POrder d T := { meet : T -> T -> T; meetC : commutative meet; meetA : associative meet; le_def : forall x y, (x <= y) = (meet x y == x); }. # [short(type="meetSemiLatticeType") ] HB.structure Definition MeetSemiLattice d := { T of POrder_isMeetSemiLattice d T & POrder d T }.

#[key="T"]
HB.mixin Record POrder_isLattice d (T : Type) of POrder d T := {
  meet : T T T;
  join : T T T;
  meetC : commutative meet;
  joinC : commutative join;
  meetA : associative meet;
  joinA : associative join;
  joinKI : y x, meet x (join x y) = x;
  meetKU : y x, join x (meet x y) = x;
  leEmeet : x y, (x y) = (meet x y == x);
}.
HB.builders Context d T of POrder_isLattice d T. Let le_defU : forall x y, (x <= y) = (join x y == y). Proof. Admitted. HB.instance Definition _ := @POrder_isMeetSemiLattice.Build d T meet meetC meetA le_def. HB.instance Definition _ := @POrder_isJoinSemiLattice.Build d T join joinC joinA le_defU. HB.end.

#[short(type="latticeType")]
HB.structure Definition Lattice d :=
  { T of POrder_isLattice d T & POrder d T }.

Module LatticeExports.
#[deprecated(since="mathcomp 2.0.0", note="Use Lattice.clone instead.")]
Notation "[ 'latticeType' 'of' T 'for' cT ]" := (Lattice.clone _ T%type cT)
  (at level 0, format "[ 'latticeType' 'of' T 'for' cT ]") : form_scope.
#[deprecated(since="mathcomp 2.0.0", note="Use Lattice.clone instead.")]
Notation "[ 'latticeType' 'of' T 'for' cT 'with' disp ]" :=
  (Lattice.clone disp T%type cT)
  (at level 0, format "[ 'latticeType' 'of' T 'for' cT 'with' disp ]") :
  form_scope.
#[deprecated(since="mathcomp 2.0.0", note="Use Lattice.clone instead.")]
Notation "[ 'latticeType' 'of' T ]" := (Lattice.clone _ T%type _)
  (at level 0, format "[ 'latticeType' 'of' T ]") : form_scope.
#[deprecated(since="mathcomp 2.0.0", note="Use Lattice.clone instead.")]
Notation "[ 'latticeType' 'of' T 'with' disp ]" := (Lattice.clone disp T%type _)
  (at level 0, format "[ 'latticeType' 'of' T 'with' disp ]") : form_scope.
End LatticeExports.

Section LatticeDef.
Context {disp : unit} {T : latticeType disp}.

Variant lel_xor_gt (x y : T) :
  T T T T T T T T bool bool Set :=
  | LelNotGt of x y : lel_xor_gt x y x x y y x x y y true false
  | GtlNotLe of y < x : lel_xor_gt x y y y x x y y x x false true.

Variant ltl_xor_ge (x y : T) :
  T T T T T T T T bool bool Set :=
  | LtlNotGe of x < y : ltl_xor_ge x y x x y y x x y y false true
  | GelNotLt of y x : ltl_xor_ge x y y y x x y y x x true false.

Variant comparel (x y : T) :
   T T T T T T T T
   bool bool bool bool bool bool Set :=
  | ComparelLt of x < y : comparel x y
    x x y y x x y y false false false true false true
  | ComparelGt of y < x : comparel x y
    y y x x y y x x false false true false true false
  | ComparelEq of x = y : comparel x y
    x x x x x x x x true true true true false false.

Variant incomparel (x y : T) :
  T T T T T T T T
  bool bool bool bool bool bool bool bool Set :=
  | InComparelLt of x < y : incomparel x y
    x x y y x x y y false false false true false true true true
  | InComparelGt of y < x : incomparel x y
    y y x x y y x x false false true false true false true true
  | InComparel of x >< y : incomparel x y
    x y y x (meet y x) (meet x y) (join y x) (join x y)
    false false false false false false false false
  | InComparelEq of x = y : incomparel x y
    x x x x x x x x true true true true false false true true.

End LatticeDef.

Module LatticeSyntax.

Notation "x `&` y" := (meet x y) : order_scope.
Notation "x `|` y" := (join x y) : order_scope.

End LatticeSyntax.

#[key="T"]
HB.mixin Record hasBottom d (T : Type) of POrder d T := {
  bottom : T;
  le0x : x, bottom x;
}.
#[short(type="bPOrderType")]
HB.structure Definition BPOrder d := { T of hasBottom d T & POrder d T }.
#[short(type="bLatticeType")]
HB.structure Definition BLattice d := { T of hasBottom d T & Lattice d T }.

Module BLatticeExports.
#[deprecated(since="mathcomp 2.0.0", note="Use BLattice.clone instead.")]
Notation "[ 'bLatticeType' 'of' T 'for' cT ]" := (BLattice.clone _ T%type cT)
  (at level 0, format "[ 'bLatticeType' 'of' T 'for' cT ]") : form_scope.
#[deprecated(since="mathcomp 2.0.0", note="Use BLattice.clone instead.")]
Notation "[ 'bLatticeType' 'of' T ]" := (BLattice.clone _ T%type _)
  (at level 0, format "[ 'bLatticeType' 'of' T ]") : form_scope.
End BLatticeExports.

Module BLatticeSyntax.
Notation "0%O" := bottom (only parsing). (* deprecated in 1.17.0 *)
Notation "\bot" := bottom : order_scope.

Notation "\join_ ( i <- r | P ) F" :=
  (\big[@join _ _ / \bot]_(i <- r | P%B) F%O) : order_scope.
Notation "\join_ ( i <- r ) F" :=
  (\big[@join _ _ / \bot]_(i <- r) F%O) : order_scope.
Notation "\join_ ( i | P ) F" :=
  (\big[@join _ _ / \bot]_(i | P%B) F%O) : order_scope.
Notation "\join_ i F" :=
  (\big[@join _ _ / \bot]_i F%O) : order_scope.
Notation "\join_ ( i : I | P ) F" :=
  (\big[@join _ _ / \bot]_(i : I | P%B) F%O) (only parsing) : order_scope.
Notation "\join_ ( i : I ) F" :=
  (\big[@join _ _ / \bot]_(i : I) F%O) (only parsing) : order_scope.
Notation "\join_ ( m <= i < n | P ) F" :=
  (\big[@join _ _ / \bot]_(m i < n | P%B) F%O) : order_scope.
Notation "\join_ ( m <= i < n ) F" :=
  (\big[@join _ _ / \bot]_(m i < n) F%O) : order_scope.
Notation "\join_ ( i < n | P ) F" :=
  (\big[@join _ _ / \bot]_(i < n | P%B) F%O) : order_scope.
Notation "\join_ ( i < n ) F" :=
  (\big[@join _ _ / \bot]_(i < n) F%O) : order_scope.
Notation "\join_ ( i 'in' A | P ) F" :=
  (\big[@join _ _ / \bot]_(i in A | P%B) F%O) : order_scope.
Notation "\join_ ( i 'in' A ) F" :=
  (\big[@join _ _ / \bot]_(i in A) F%O) : order_scope.

End BLatticeSyntax.

#[key="T"]
HB.mixin Record hasTop d (T : Type) of POrder d T := {
  top : T;
  lex1 : x, x top;
}.
#[short(type="tPOrderType")]
HB.structure Definition TPOrder d := { T of hasTop d T & POrder d T }.
#[short(type="tbPOrderType")]
HB.structure Definition TBPOrder d := { T of hasTop d T & BPOrder d T }.
#[short(type="tLatticeType")]
HB.structure Definition TLattice d := { T of hasTop d T & Lattice d T }.
#[short(type="tbLatticeType")]
HB.structure Definition TBLattice d := { T of BLattice d T & TLattice d T }.

Module TLatticeSyntax.

Notation "1%O" := top (only parsing). (* deprecated in 1.17.0 *)
Notation "\top" := top : order_scope.

Notation "\meet_ ( i <- r | P ) F" :=
  (\big[meet / \top]_(i <- r | P%B) F%O) : order_scope.
Notation "\meet_ ( i <- r ) F" :=
  (\big[meet / \top]_(i <- r) F%O) : order_scope.
Notation "\meet_ ( i | P ) F" :=
  (\big[meet / \top]_(i | P%B) F%O) : order_scope.
Notation "\meet_ i F" :=
  (\big[meet / \top]_i F%O) : order_scope.
Notation "\meet_ ( i : I | P ) F" :=
  (\big[meet / \top]_(i : I | P%B) F%O) (only parsing) : order_scope.
Notation "\meet_ ( i : I ) F" :=
  (\big[meet / \top]_(i : I) F%O) (only parsing) : order_scope.
Notation "\meet_ ( m <= i < n | P ) F" :=
 (\big[meet / \top]_(m i < n | P%B) F%O) : order_scope.
Notation "\meet_ ( m <= i < n ) F" :=
 (\big[meet / \top]_(m i < n) F%O) : order_scope.
Notation "\meet_ ( i < n | P ) F" :=
 (\big[meet / \top]_(i < n | P%B) F%O) : order_scope.
Notation "\meet_ ( i < n ) F" :=
 (\big[meet / \top]_(i < n) F%O) : order_scope.
Notation "\meet_ ( i 'in' A | P ) F" :=
 (\big[meet / \top]_(i in A | P%B) F%O) : order_scope.
Notation "\meet_ ( i 'in' A ) F" :=
 (\big[meet / \top]_(i in A) F%O) : order_scope.

End TLatticeSyntax.

#[key="T"]
HB.mixin Record Lattice_Meet_isDistrLattice d (T : Type) of Lattice d T := {
  meetUl : @left_distributive T T meet join;
}.
#[short(type="distrLatticeType")]
HB.structure Definition DistrLattice d :=
  { T of Lattice_Meet_isDistrLattice d T & Lattice d T }.

#[short(type="bDistrLatticeType")]
HB.structure Definition BDistrLattice d :=
  { T of hasBottom d T & DistrLattice d T}.

Module BDistrLatticeExports.
#[deprecated(since="mathcomp 2.0.0", note="Use BDistrLattice.clone instead.")]
Notation "[ 'bDistrLatticeType' 'of' T ]" := (BDistrLattice.clone _ T%type _)
  (at level 0, format "[ 'bDistrLatticeType' 'of' T ]") : form_scope.
End BDistrLatticeExports.

#[short(type="tbDistrLatticeType")]
HB.structure Definition TBDistrLattice d :=
  { T of TBLattice d T & BDistrLattice d T }.

Module TBDistrLatticeExports.
#[deprecated(since="mathcomp 2.0.0", note="Use TBDistrLattice.clone instead.")]
Notation "[ 'tbDistrLatticeType' 'of' T ]" := (TBDistrLattice.clone _ T%type _)
  (at level 0, format "[ 'tbDistrLatticeType' 'of' T ]") : form_scope.
End TBDistrLatticeExports.

#[key="T"]
HB.mixin Record hasRelativeComplement d (T : Type) of BDistrLattice d T := {
  diff : T T T;
  diffKI : x y, y `&` diff x y = bottom;
  joinIB : x y, (x `&` y) `|` diff x y = x
}.

#[short(type="cbDistrLatticeType")]
HB.structure Definition CBDistrLattice d :=
  { T of hasRelativeComplement d T & BDistrLattice d T }.

#[deprecated(since="mathcomp 2.0.0", note="Use diff instead.")]
Notation sub := diff.
#[deprecated(since="mathcomp 2.0.0", note="Use diffKI instead.")]
Notation subKI := diffKI.

Module Import CBDistrLatticeSyntax.
Notation "x `\` y" := (diff x y) : order_scope.
End CBDistrLatticeSyntax.

#[key="T"]
HB.mixin Record hasComplement d (T : Type) of
         TBDistrLattice d T & CBDistrLattice d T := {
  compl : T T;
  complE : x : T, compl x = (top : T) `\` x (* FIXME? *)
}.

#[short(type="ctbDistrLatticeType")]
HB.structure Definition CTBDistrLattice d :=
  { T of hasComplement d T & TBDistrLattice d T & CBDistrLattice d T }.

Module Import CTBDistrLatticeSyntax.
Notation "~` A" := (compl A) : order_scope.
End CTBDistrLatticeSyntax.


#[short(type="orderType")]
HB.structure Definition Total d :=
  { T of DistrLattice_isTotal d T & DistrLattice d T }.

FINITE

#[short(type="finPOrderType")]
HB.structure Definition FinPOrder d := { T of Finite T & POrder d T }.

Module FinPOrderExports.
#[deprecated(since="mathcomp 2.0.0", note="Use BLattice.clone instead.")]
Notation "[ 'finPOrderType' 'of' T ]" := (FinPOrder.clone _ T%type _ )
  (at level 0, format "[ 'finPOrderType' 'of' T ]") : form_scope.
End FinPOrderExports.

#[short(type="finLatticeType")]
HB.structure Definition FinLattice d := { T of Finite T & TBLattice d T }. (* FIXME *)

Module FinLatticeExports.
#[deprecated(since="mathcomp 2.0.0", note="Use FinLattice.clone instead.")]
Notation "[ 'finLatticeType' 'of' T ]" := (FinLattice.clone _ T%type _ )
  (at level 0, format "[ 'finLatticeType' 'of' T ]") : form_scope.
End FinLatticeExports.

#[short(type="finDistrLatticeType")]
HB.structure Definition FinDistrLattice d :=
  { T of Finite T & TBDistrLattice d T }.

Module FinDistrLatticeExports.
#[deprecated(since="mathcomp 2.0.0", note="Use FinDistrLattice.clone instead.")]
Notation "[ 'finDistrLatticeType' 'of' T ]" := (FinDistrLattice.clone _ T%type _ )
  (at level 0, format "[ 'finDistrLatticeType' 'of' T ]") : form_scope.
End FinDistrLatticeExports.

#[short(type="finCDistrLatticeType")]
HB.structure Definition FinCDistrLattice d :=
  { T of Finite T & CTBDistrLattice d T }.

Module FinCDistrLatticeExports.
#[deprecated(since="mathcomp 2.0.0", note="Use FinCDistrLattice.clone instead.")]
Notation "[ 'finCDistrLatticeType' 'of' T ]" := (FinCDistrLattice.clone _ T%type _ )
  (at level 0, format "[ 'finCDistrLatticeType' 'of' T ]") : form_scope.
End FinCDistrLatticeExports.

#[short(type="finOrderType")]
HB.structure Definition FinTotal d :=
  { T of Total d T & FinDistrLattice d T }.

Module FinTotalExports.
#[deprecated(since="mathcomp 2.0.0", note="Use FinTotal.clone instead.")]
Notation "[ 'finOrderType' 'of' T ]" := (FinTotal.clone _ T%type _ )
  (at level 0, format "[ 'finOrderType' 'of' T ]") : form_scope.
End FinTotalExports.

DUAL

Definition dual T : Type := T.
Definition dual_display : unit unit.

Notation dual_le := (@le (dual_display _) _).
Notation dual_lt := (@lt (dual_display _) _).
Notation dual_comparable := (@comparable (dual_display _) _).
Notation dual_ge := (@ge (dual_display _) _).
Notation dual_gt := (@gt (dual_display _) _).
Notation dual_leif := (@leif (dual_display _) _).
Notation dual_lteif := (@lteif (dual_display _) _).
Notation dual_max := (@max (dual_display _) _).
Notation dual_min := (@min (dual_display _) _).
Notation dual_meet := (@meet (dual_display _) _).
Notation dual_join := (@join (dual_display _) _).
Notation dual_bottom := (@bottom (dual_display _) _).
Notation dual_top := (@top (dual_display _) _).

Module Import DualSyntax.

Notation "T ^d" := (dual T) (at level 2, format "T ^d") : type_scope.
Notation "<=^d%O" := dual_le : function_scope.
Notation ">=^d%O" := dual_ge : function_scope.
Notation "<^d%O" := dual_lt : function_scope.
Notation ">^d%O" := dual_gt : function_scope.
Notation "<?=^d%O" := dual_leif : function_scope.
Notation "<?<=^d%O" := dual_lteif : function_scope.
Notation ">=<^d%O" := dual_comparable : function_scope.
Notation "><^d%O" := (fun x y~~ dual_comparable x y) : function_scope.

Notation "<=^d y" := (>=^d%O y) : order_scope.
Notation "<=^d y :> T" := (<=^d (y : T)) (only parsing) : order_scope.
Notation ">=^d y" := (<=^d%O y) : order_scope.
Notation ">=^d y :> T" := (>=^d (y : T)) (only parsing) : order_scope.

Notation "<^d y" := (>^d%O y) : order_scope.
Notation "<^d y :> T" := (<^d (y : T)) (only parsing) : order_scope.
Notation ">^d y" := (<^d%O y) : order_scope.
Notation ">^d y :> T" := (>^d (y : T)) (only parsing) : order_scope.

Notation "x <=^d y" := (<=^d%O x y) : order_scope.
Notation "x <=^d y :> T" := ((x : T) <=^d (y : T)) (only parsing) : order_scope.
Notation "x >=^d y" := (y <=^d x) (only parsing) : order_scope.
Notation "x >=^d y :> T" := ((x : T) >=^d (y : T)) (only parsing) : order_scope.

Notation "x <^d y" := (<^d%O x y) : order_scope.
Notation "x <^d y :> T" := ((x : T) <^d (y : T)) (only parsing) : order_scope.
Notation "x >^d y" := (y <^d x) (only parsing) : order_scope.
Notation "x >^d y :> T" := ((x : T) >^d (y : T)) (only parsing) : order_scope.

Notation "x <=^d y <=^d z" := ((x <=^d y) && (y <=^d z)) : order_scope.
Notation "x <^d y <=^d z" := ((x <^d y) && (y <=^d z)) : order_scope.
Notation "x <=^d y <^d z" := ((x <=^d y) && (y <^d z)) : order_scope.
Notation "x <^d y <^d z" := ((x <^d y) && (y <^d z)) : order_scope.

Notation "x <=^d y ?= 'iff' C" := (<?=^d%O x y C) : order_scope.
Notation "x <=^d y ?= 'iff' C :> T" := ((x : T) <=^d (y : T) ?= iff C)
  (only parsing) : order_scope.

Notation "x <^d y ?<= 'if' C" := (<?<=^d%O x y C) : order_scope.
Notation "x <^d y ?<= 'if' C :> T" := ((x : T) <^d (y : T) ?<= if C)
  (only parsing) : order_scope.

Notation ">=<^d x" := (>=<^d%O x) : order_scope.
Notation ">=<^d y :> T" := (>=<^d (y : T)) (only parsing) : order_scope.
Notation "x >=<^d y" := (>=<^d%O x y) : order_scope.

Notation "><^d y" := [pred x | ~~ dual_comparable x y] : order_scope.
Notation "><^d y :> T" := (><^d (y : T)) (only parsing) : order_scope.
Notation "x ><^d y" := (~~ (><^d%O x y)) : order_scope.

Notation "x `&^d` y" := (dual_meet x y) : order_scope.
Notation "x `|^d` y" := (dual_join x y) : order_scope.

Notation "0^d%O" := dual_bottom (only parsing). (* deprecated in 1.17.0 *)
Notation "1^d%O" := dual_top (only parsing). (* deprecated in 1.17.0 *)
Notation "\bot^d" := dual_bottom : order_scope.
Notation "\top^d" := dual_top : order_scope.

The following Local Notations are here to define the \join^d_ and \meet^d_ notations later. Do not remove them.

Notation "\join^d_ ( i <- r | P ) F" :=
  (\big[join / \bot]_(i <- r | P%B) F%O) : order_scope.
Notation "\join^d_ ( i <- r ) F" :=
  (\big[join / \bot]_(i <- r) F%O) : order_scope.
Notation "\join^d_ ( i | P ) F" :=
  (\big[join / \bot]_(i | P%B) F%O) : order_scope.
Notation "\join^d_ i F" :=
  (\big[join / \bot]_i F%O) : order_scope.
Notation "\join^d_ ( i : I | P ) F" :=
  (\big[join / \bot]_(i : I | P%B) F%O) (only parsing) : order_scope.
Notation "\join^d_ ( i : I ) F" :=
  (\big[join / \bot]_(i : I) F%O) (only parsing) : order_scope.
Notation "\join^d_ ( m <= i < n | P ) F" :=
 (\big[join / \bot]_(m i < n | P%B) F%O) : order_scope.
Notation "\join^d_ ( m <= i < n ) F" :=
 (\big[join / \bot]_(m i < n) F%O) : order_scope.
Notation "\join^d_ ( i < n | P ) F" :=
 (\big[join / \bot]_(i < n | P%B) F%O) : order_scope.
Notation "\join^d_ ( i < n ) F" :=
 (\big[join / \bot]_(i < n) F%O) : order_scope.
Notation "\join^d_ ( i 'in' A | P ) F" :=
 (\big[join / \bot]_(i in A | P%B) F%O) : order_scope.
Notation "\join^d_ ( i 'in' A ) F" :=
 (\big[join / \bot]_(i in A) F%O) : order_scope.

Notation "\meet^d_ ( i <- r | P ) F" :=
  (\big[meet / \top]_(i <- r | P%B) F%O) : order_scope.
Notation "\meet^d_ ( i <- r ) F" :=
  (\big[meet / \top]_(i <- r) F%O) : order_scope.
Notation "\meet^d_ ( i | P ) F" :=
  (\big[meet / \top]_(i | P%B) F%O) : order_scope.
Notation "\meet^d_ i F" :=
  (\big[meet / \top]_i F%O) : order_scope.
Notation "\meet^d_ ( i : I | P ) F" :=
  (\big[meet / \top]_(i : I | P%B) F%O) (only parsing) : order_scope.
Notation "\meet^d_ ( i : I ) F" :=
  (\big[meet / \top]_(i : I) F%O) (only parsing) : order_scope.
Notation "\meet^d_ ( m <= i < n | P ) F" :=
 (\big[meet / \top]_(m i < n | P%B) F%O) : order_scope.
Notation "\meet^d_ ( m <= i < n ) F" :=
 (\big[meet / \top]_(m i < n) F%O) : order_scope.
Notation "\meet^d_ ( i < n | P ) F" :=
 (\big[meet / \top]_(i < n | P%B) F%O) : order_scope.
Notation "\meet^d_ ( i < n ) F" :=
 (\big[meet / \top]_(i < n) F%O) : order_scope.
Notation "\meet^d_ ( i 'in' A | P ) F" :=
 (\big[meet / \top]_(i in A | P%B) F%O) : order_scope.
Notation "\meet^d_ ( i 'in' A ) F" :=
 (\big[meet / \top]_(i in A) F%O) : order_scope.

End DualSyntax.

THEORY

Module Import POrderTheory.
Section POrderTheory.

Context {disp : unit} {T : porderType disp}.

Implicit Types (x y : T) (s : seq T).

Lemma geE x y : ge x y = (y x).
Lemma gtE x y : gt x y = (y < x).

Lemma lexx (x : T) : x x.
Hint Resolve lexx : core.

Definition le_refl : reflexive le := lexx.
Definition ge_refl : reflexive ge := lexx.
Hint Resolve le_refl : core.

Lemma le_anti: antisymmetric (<=%O : rel T).

Lemma ge_anti: antisymmetric (>=%O : rel T).

Lemma le_trans: transitive (<=%O : rel T).

Lemma ge_trans: transitive (>=%O : rel T).

Lemma le_le_trans x y z t : z x y t x y z t.

Lemma lt_def x y: (x < y) = (y != x) && (x y).

Lemma lt_neqAle x y: (x < y) = (x != y) && (x y).

Lemma ltxx x: x < x = false.

Definition lt_irreflexive : irreflexive lt := ltxx.
Hint Resolve lt_irreflexive : core.

Definition ltexx := (lexx, ltxx).

Lemma le_eqVlt x y: (x y) = (x == y) || (x < y).

Lemma lt_eqF x y: x < y x == y = false.

Lemma gt_eqF x y : y < x x == y = false.

Lemma eq_le x y: (x == y) = (x y x).

Lemma ltW x y: x < y x y.

Lemma lt_le_trans y x z: x < y y z x < z.

Lemma lt_trans: transitive (<%O : rel T).

Lemma le_lt_trans y x z: x y y < z x < z.

Lemma lt_nsym x y : x < y y < x False.

Lemma lt_asym x y : x < y < x = false.

Lemma le_gtF x y: x y y < x = false.

Lemma lt_geF x y : (x < y) y x = false.

Definition lt_gtF x y hxy := le_gtF (@ltW x y hxy).

Lemma lt_leAnge x y : (x < y) = (x y) && ~~ (y x).

Lemma lt_le_asym x y : x < y x = false.

Lemma le_lt_asym x y : x y < x = false.

Definition lte_anti := (=^~ eq_le, lt_asym, lt_le_asym, le_lt_asym).

Lemma le_path_min x s : path <=%O x s all ( x) s.

Lemma lt_path_min x s : path <%O x s all (> x) s.

Lemma le_path_sortedE x s : path <=%O x s = all ( x) s && sorted <=%O s.

Lemma lt_path_sortedE x s : path <%O x s = all (> x) s && sorted <%O s.

Lemma le_sorted_pairwise s : sorted <=%O s = pairwise <=%O s.

Lemma lt_sorted_pairwise s : sorted <%O s = pairwise <%O s.

Lemma le_path_pairwise x s : path <=%O x s = pairwise <=%O (x :: s).

Lemma lt_path_pairwise x s : path <%O x s = pairwise <%O (x :: s).

Lemma lt_sorted_uniq_le s : sorted <%O s = uniq s && sorted <=%O s.

Lemma le_sorted_mask m s : sorted <=%O s sorted <=%O (mask m s).

Lemma lt_sorted_mask m s : sorted <%O s sorted <%O (mask m s).

Lemma le_sorted_filter a s : sorted <=%O s sorted <=%O (filter a s).

Lemma lt_sorted_filter a s : sorted <%O s sorted <%O (filter a s).

Lemma le_path_mask x m s : path <=%O x s path <=%O x (mask m s).

Lemma lt_path_mask x m s : path <%O x s path <%O x (mask m s).

Lemma le_path_filter x a s : path <=%O x s path <=%O x (filter a s).

Lemma lt_path_filter x a s : path <%O x s path <%O x (filter a s).

Lemma le_sorted_ltn_nth (x0 : T) (s : seq T) : sorted <=%O s
 {in [pred n | (n < size s)%N] &,
    {homo nth x0 s : i j / (i < j)%N >-> i j}}.

Lemma le_sorted_leq_nth (x0 : T) (s : seq T) : sorted <=%O s
  {in [pred n | (n < size s)%N] &,
    {homo nth x0 s : i j / (i j)%N >-> i j}}.

Lemma lt_sorted_leq_nth (x0 : T) (s : seq T) : sorted <%O s
  {in [pred n | (n < size s)%N] &,
    {mono nth x0 s : i j / (i j)%N >-> i j}}.

Lemma lt_sorted_ltn_nth (x0 : T) (s : seq T) : sorted <%O s
  {in [pred n | (n < size s)%N] &,
    {mono nth x0 s : i j / (i < j)%N >-> i < j}}.

Lemma subseq_le_path x s1 s2 : subseq s1 s2 path <=%O x s2 path <=%O x s1.

Lemma subseq_lt_path x s1 s2 : subseq s1 s2 path <%O x s2 path <%O x s1.

Lemma subseq_le_sorted s1 s2 : subseq s1 s2 sorted <=%O s2 sorted <=%O s1.

Lemma subseq_lt_sorted s1 s2 : subseq s1 s2 sorted <%O s2 sorted <%O s1.

Lemma lt_sorted_uniq s : sorted <%O s uniq s.

Lemma lt_sorted_eq s1 s2 :
  sorted <%O s1 sorted <%O s2 s1 =i s2 s1 = s2.

Lemma le_sorted_eq s1 s2 :
  sorted <=%O s1 sorted <=%O s2 perm_eq s1 s2 s1 = s2.

Lemma filter_lt_nth x0 s i : sorted <%O s (i < size s)%N
  [seq x <- s | x < nth x0 s i] = take i s.

Lemma count_lt_nth x0 s i : sorted <%O s (i < size s)%N
  count (< nth x0 s i) s = i.

Lemma filter_le_nth x0 s i : sorted <%O s (i < size s)%N
  [seq x <- s | x nth x0 s i] = take i.+1 s.

Lemma count_le_nth x0 s i : sorted <%O s (i < size s)%N
  count ( nth x0 s i) s = i.+1.

Lemma count_lt_le_mem x s : (count (< x) s < count ( x) s)%N = (x \in s).

Lemma sorted_filter_lt x s :
  sorted <=%O s [seq y <- s | y < x] = take (count (< x) s) s.

Lemma sorted_filter_le x s :
  sorted <=%O s [seq y <- s | y x] = take (count ( x) s) s.

Lemma nth_count_le x x0 s i : sorted <=%O s
  (i < count ( x) s)%N nth x0 s i x.

Lemma nth_count_lt x x0 s i : sorted <=%O s
  (i < count (< x) s)%N nth x0 s i < x.

Lemma sort_le_id s : sorted <=%O s sort <=%O s = s.

Lemma sort_lt_id s : sorted <%O s sort <%O s = s.

Lemma comparable_leNgt x y : x >=< y (x y) = ~~ (y < x).

Lemma comparable_ltNge x y : x >=< y (x < y) = ~~ (y x).

Lemma comparable_ltgtP x y : x >=< y
  compare x y (min y x) (min x y) (max y x) (max x y)
  (y == x) (x == y) (x y) (x y) (x > y) (x < y).

Lemma comparable_leP x y : x >=< y
  le_xor_gt x y (min y x) (min x y) (max y x) (max x y) (x y) (y < x).

Lemma comparable_ltP x y : x >=< y
  lt_xor_ge x y (min y x) (min x y) (max y x) (max x y) (y x) (x < y).

Lemma comparable_sym x y : (y >=< x) = (x >=< y).

Lemma comparablexx x : x >=< x.

Lemma incomparable_eqF x y : (x >< y) (x == y) = false.

Lemma incomparable_leF x y : (x >< y) (x y) = false.

Lemma incomparable_ltF x y : (x >< y) (x < y) = false.

Lemma comparableP x y : incompare x y
  (min y x) (min x y) (max y x) (max x y)
  (y == x) (x == y) (x y) (x y) (x > y) (x < y)
  (y >=< x) (x >=< y).

Lemma le_comparable (x y : T) : x y x >=< y.

Lemma lt_comparable (x y : T) : x < y x >=< y.

Lemma ge_comparable (x y : T) : y x x >=< y.

Lemma gt_comparable (x y : T) : y < x x >=< y.

leif

Lemma leifP x y C : reflect (x y ?= iff C) (if C then x == y else x < y).

Lemma leif_refl x C : reflect (x x ?= iff C) C.

Lemma leif_trans x1 x2 x3 C12 C23 :
  x1 x2 ?= iff C12 x2 x3 ?= iff C23 x1 x3 ?= iff C12 && C23.

Lemma leif_le x y : x y x y ?= iff (x y).

Lemma leif_eq x y : x y x y ?= iff (x == y).

Lemma ge_leif x y C : x y ?= iff C (y x) = C.

Lemma lt_leif x y C : x y ?= iff C (x < y) = ~~ C.

Lemma ltNleif x y C : x y ?= iff ~~ C (x < y) = C.

Lemma eq_leif x y C : x y ?= iff C (x == y) = C.

Lemma eqTleif x y C : x y ?= iff C C x = y.

lteif

Lemma lteif_trans x y z C1 C2 :
  x < y ?<= if C1 y < z ?<= if C2 x < z ?<= if C1 && C2.

Lemma lteif_anti C1 C2 x y :
  (x < y ?<= if C1) && (y < x ?<= if C2) = C1 && C2 && (x == y).

Lemma lteifxx x C : (x < x ?<= if C) = C.

Lemma lteifNF x y C : y < x ?<= if ~~ C x < y ?<= if C = false.

Lemma lteifS x y C : x < y x < y ?<= if C.

Lemma lteifT x y : x < y ?<= if true = (x y).

Lemma lteifF x y : x < y ?<= if false = (x < y).

Lemma lteif_orb x y : {morph lteif x y : p q / p || q}.

Lemma lteif_andb x y : {morph lteif x y : p q / p && q}.

Lemma lteif_imply C1 C2 x y : C1 ==> C2 x < y ?<= if C1 x < y ?<= if C2.

Lemma lteifW C x y : x < y ?<= if C x y.

Lemma ltrW_lteif C x y : x < y x < y ?<= if C.

Lemma lteifN C x y : x < y ?<= if ~~ C ~~ (y < x ?<= if C).

min and max

Lemma minElt x y : min x y = if x < y then x else y.
Lemma maxElt x y : max x y = if x < y then y else x.

Lemma minEle x y : min x y = if x y then x else y.

Lemma maxEle x y : max x y = if x y then y else x.

Lemma comparable_minEgt x y : x >=< y min x y = if x > y then y else x.
Lemma comparable_maxEgt x y : x >=< y max x y = if x > y then x else y.
Lemma comparable_minEge x y : x >=< y min x y = if x y then y else x.
Lemma comparable_maxEge x y : x >=< y max x y = if x y then x else y.

Lemma min_l x y : x y min x y = x.
Lemma min_r x y : y x min x y = y.
Lemma max_l x y : y x max x y = x.
Lemma max_r x y : x y max x y = y.

Lemma minxx : idempotent (min : T T T).

Lemma maxxx : idempotent (max : T T T).

Lemma eq_minl x y : (min x y == x) = (x y).

Lemma eq_maxr x y : (max x y == y) = (x y).

Lemma min_idPl x y : reflect (min x y = x) (x y).

Lemma max_idPr x y : reflect (max x y = y) (x y).

Lemma min_minKx x y : min (min x y) y = min x y.

Lemma min_minxK x y : min x (min x y) = min x y.

Lemma max_maxKx x y : max (max x y) y = max x y.

Lemma max_maxxK x y : max x (max x y) = max x y.

Lemma comparable_minl z : {in >=< z &, x y, min x y >=< z}.

Lemma comparable_minr z : {in >=<%O z &, x y, z >=< min x y}.

Lemma comparable_maxl z : {in >=< z &, x y, max x y >=< z}.

Lemma comparable_maxr z : {in >=<%O z &, x y, z >=< max x y}.

Section Comparable2.
Variables (z x y : T) (cmp_xy : x >=< y).

Lemma comparable_minC : min x y = min y x.

Lemma comparable_maxC : max x y = max y x.

Lemma comparable_eq_minr : (min x y == y) = (y x).

Lemma comparable_eq_maxl : (max x y == x) = (y x).

Lemma comparable_min_idPr : reflect (min x y = y) (y x).

Lemma comparable_max_idPl : reflect (max x y = x) (y x).

Lemma comparable_le_min : (z min x y) = (z x) && (z y).

Lemma comparable_ge_min : (min x y z) = (x z) || (y z).

Lemma comparable_lt_min : (z < min x y) = (z < x) && (z < y).

Lemma comparable_gt_min : (min x y < z) = (x < z) || (y < z).

Lemma comparable_le_max : (z max x y) = (z x) || (z y).

Lemma comparable_ge_max : (max x y z) = (x z) && (y z).

Lemma comparable_lt_max : (z < max x y) = (z < x) || (z < y).

Lemma comparable_gt_max : (max x y < z) = (x < z) && (y < z).

Lemma comparable_minxK : max (min x y) y = y.

Lemma comparable_minKx : max x (min x y) = x.

Lemma comparable_maxxK : min (max x y) y = y.

Lemma comparable_maxKx : min x (max x y) = x.

Lemma comparable_lteifNE C : x >=< y x < y ?<= if ~~ C = ~~ (y < x ?<= if C).

Lemma comparable_lteif_minr C :
  (z < Order.min x y ?<= if C) = (z < x ?<= if C) && (z < y ?<= if C).

Lemma comparable_lteif_minl C :
  (Order.min x y < z ?<= if C) = (x < z ?<= if C) || (y < z ?<= if C).

Lemma comparable_lteif_maxr C :
  (z < Order.max x y ?<= if C) = (z < x ?<= if C) || (z < y ?<= if C).

Lemma comparable_lteif_maxl C :
  (Order.max x y < z ?<= if C) = (x < z ?<= if C) && (y < z ?<= if C).

End Comparable2.

Section Comparable3.
Variables (x y z : T) (cmp_xy : x >=< y) (cmp_xz : x >=< z) (cmp_yz : y >=< z).
Let P := comparableP.

Lemma comparable_minA : min x (min y z) = min (min x y) z.

Lemma comparable_maxA : max x (max y z) = max (max x y) z.

Lemma comparable_max_minl : max (min x y) z = min (max x z) (max y z).

Lemma comparable_min_maxl : min (max x y) z = max (min x z) (min y z).

End Comparable3.

Lemma comparable_minAC x y z : x >=< y x >=< z y >=< z
  min (min x y) z = min (min x z) y.

Lemma comparable_maxAC x y z : x >=< y x >=< z y >=< z
  max (max x y) z = max (max x z) y.

Lemma comparable_minCA x y z : x >=< y x >=< z y >=< z
  min x (min y z) = min y (min x z).

Lemma comparable_maxCA x y z : x >=< y x >=< z y >=< z
  max x (max y z) = max y (max x z).

Lemma comparable_minACA x y z t :
    x >=< y x >=< z x >=< t y >=< z y >=< t z >=< t
  min (min x y) (min z t) = min (min x z) (min y t).

Lemma comparable_maxACA x y z t :
    x >=< y x >=< z x >=< t y >=< z y >=< t z >=< t
  max (max x y) (max z t) = max (max x z) (max y t).

Lemma comparable_max_minr x y z : x >=< y x >=< z y >=< z
  max x (min y z) = min (max x y) (max x z).

Lemma comparable_min_maxr x y z : x >=< y x >=< z y >=< z
  min x (max y z) = max (min x y) (min x z).

Section ArgExtremum.

Context (I : finType) (i0 : I) (P : {pred I}) (F : I T) (Pi0 : P i0).
Hypothesis F_comparable : {in P &, i j, F i >=< F j}.

Lemma comparable_arg_minP: extremum_spec <=%O P F (arg_min i0 P F).

Lemma comparable_arg_maxP: extremum_spec >=%O P F (arg_max i0 P F).

End ArgExtremum.

monotonicity

Lemma mono_in_leif (A : {pred T}) (f : T T) C :
   {in A &, {mono f : x y / x y}}
  {in A &, x y, (f x f y ?= iff C) = (x y ?= iff C)}.

Lemma mono_leif (f : T T) C :
    {mono f : x y / x y}
   x y, (f x f y ?= iff C) = (x y ?= iff C).

Lemma nmono_in_leif (A : {pred T}) (f : T T) C :
    {in A &, {mono f : x y /~ x y}}
  {in A &, x y, (f x f y ?= iff C) = (y x ?= iff C)}.

Lemma nmono_leif (f : T T) C : {mono f : x y /~ x y}
   x y, (f x f y ?= iff C) = (y x ?= iff C).

Lemma comparable_bigl x x0 op I (P : pred I) F (s : seq I) :
  {in >=< x &, y z, op y z >=< x} x0 >=< x
  {in P, i, F i >=< x} \big[op/x0]_(i <- s | P i) F i >=< x.

Lemma comparable_bigr x x0 op I (P : pred I) F (s : seq I) :
  {in >=<%O x &, y z, x >=< op y z} x >=< x0
  {in P, i, x >=< F i} x >=< \big[op/x0]_(i <- s | P i) F i.

Section bigminmax.

Variables (I : Type) (r : seq I) (f : I T) (x0 x : T) (P : pred I).

Lemma bigmax_le : x0 x ( i, P i f i x)
  \big[max/x0]_(i <- r | P i) f i x.

Lemma bigmax_lt : x0 < x ( i, P i f i < x)
  \big[max/x0]_(i <- r | P i) f i < x.

Lemma lt_bigmin : x < x0 ( i, P i x < f i)
  x < \big[min/x0]_(i <- r | P i) f i.

Lemma le_bigmin : x x0 ( i, P i x f i)
  x \big[min/x0]_(i <- r | P i) f i.

End bigminmax.

End POrderTheory.
#[global] Hint Resolve comparable_minr comparable_minl : core.
#[global] Hint Resolve comparable_maxr comparable_maxl : core.

Section ContraTheory.
Context {disp1 disp2 : unit} {T1 : porderType disp1} {T2 : porderType disp2}.
Implicit Types (x y : T1) (z t : T2) (b : bool) (m n : nat) (P : Prop).

Lemma comparable_contraTle b x y : x >=< y (y < x ~~ b) (b x y).

Lemma comparable_contraTlt b x y : x >=< y (y x ~~ b) (b x < y).

Lemma comparable_contraPle P x y : x >=< y (y < x ¬ P) (P x y).

Lemma comparable_contraPlt P x y : x >=< y (y x ¬ P) (P x < y).

Lemma comparable_contraNle b x y : x >=< y (y < x b) (~~ b x y).

Lemma comparable_contraNlt b x y : x >=< y (y x b) (~~ b x < y).

Lemma comparable_contra_not_le P x y : x >=< y (y < x P) (¬ P x y).

Lemma comparable_contra_not_lt P x y : x >=< y (y x P) (¬ P x < y).

Lemma comparable_contraFle b x y : x >=< y (y < x b) (b = false x y).

Lemma comparable_contraFlt b x y : x >=< y (y x b) (b = false x < y).

Lemma contra_leT b x y : (~~ b x < y) (y x b).

Lemma contra_ltT b x y : (~~ b x y) (y < x b).

Lemma contra_leN b x y : (b x < y) (y x ~~ b).

Lemma contra_ltN b x y : (b x y) (y < x ~~ b).

Lemma contra_le_not P x y : (P x < y) (y x ¬ P).

Lemma contra_lt_not P x y : (P x y) (y < x ¬ P).

Lemma contra_leF b x y : (b x < y) (y x b = false).

Lemma contra_ltF b x y : (b x y) (y < x b = false).

Lemma comparable_contra_leq_le m n x y : x >=< y
  (y < x (n < m)%N) ((m n)%N x y).

Lemma comparable_contra_leq_lt m n x y : x >=< y
  (y x (n < m)%N) ((m n)%N x < y).

Lemma comparable_contra_ltn_le m n x y : x >=< y
  (y < x (n m)%N) ((m < n)%N x y).

Lemma comparable_contra_ltn_lt m n x y : x >=< y
  (y x (n m)%N) ((m < n)%N x < y).

Lemma contra_le_leq x y m n : ((n < m)%N y < x) (x y (m n)%N).

Lemma contra_le_ltn x y m n : ((n m)%N y < x) (x y (m < n)%N).

Lemma contra_lt_leq x y m n : ((n < m)%N y x) (x < y (m n)%N).

Lemma contra_lt_ltn x y m n : ((n m)%N y x) (x < y (m < n)%N).

Lemma comparable_contra_le x y z t : z >=< t
  (t < z y < x) (x y z t).

Lemma comparable_contra_le_lt x y z t : z >=< t
  (t z y < x) (x y z < t).

Lemma comparable_contra_lt_le x y z t : z >=< t
  (t < z y x) (x < y z t).

Lemma comparable_contra_lt x y z t : z >=< t
 (t z y x) (x < y z < t).

End ContraTheory.

Section POrderMonotonyTheory.

Context {disp disp' : unit}.
Context {T : porderType disp} {T' : porderType disp'}.
Implicit Types (m n p : nat) (x y z : T) (u v w : T').
Variables (D D' : {pred T}) (f : T T').

Let leT_anti := @le_anti _ T.
Let leT'_anti := @le_anti _ T'.
Hint Resolve lexx lt_neqAle lt_def : core.

Let ge_antiT : antisymmetric (>=%O : rel T).

Lemma ltW_homo : {homo f : x y / x < y} {homo f : x y / x y}.

Lemma ltW_nhomo : {homo f : x y /~ x < y} {homo f : x y /~ x y}.

Lemma inj_homo_lt :
  injective f {homo f : x y / x y} {homo f : x y / x < y}.

Lemma inj_nhomo_lt :
  injective f {homo f : x y /~ x y} {homo f : x y /~ x < y}.

Lemma inc_inj : {mono f : x y / x y} injective f.

Lemma dec_inj : {mono f : x y /~ x y} injective f.

Lemma leW_mono : {mono f : x y / x y} {mono f : x y / x < y}.

Lemma leW_nmono : {mono f : x y /~ x y} {mono f : x y /~ x < y}.

Monotony in D D'
Lemma ltW_homo_in :
  {in D & D', {homo f : x y / x < y}} {in D & D', {homo f : x y / x y}}.

Lemma ltW_nhomo_in :
  {in D & D', {homo f : x y /~ x < y}} {in D & D', {homo f : x y /~ x y}}.

Lemma inj_homo_lt_in :
    {in D & D', injective f} {in D & D', {homo f : x y / x y}}
  {in D & D', {homo f : x y / x < y}}.

Lemma inj_nhomo_lt_in :
    {in D & D', injective f} {in D & D', {homo f : x y /~ x y}}
  {in D & D', {homo f : x y /~ x < y}}.

Lemma inc_inj_in : {in D &, {mono f : x y / x y}}
   {in D &, injective f}.

Lemma dec_inj_in :
  {in D &, {mono f : x y /~ x y}} {in D &, injective f}.

Lemma leW_mono_in :
  {in D &, {mono f : x y / x y}} {in D &, {mono f : x y / x < y}}.

Lemma leW_nmono_in :
  {in D &, {mono f : x y /~ x y}} {in D &, {mono f : x y /~ x < y}}.

End POrderMonotonyTheory.

End POrderTheory.

#[global] Hint Resolve lexx le_refl ltxx lt_irreflexive ltW lt_eqF : core.

Arguments leifP {disp T x y C}.
Arguments leif_refl {disp T x C}.
Arguments mono_in_leif [disp T A f C].
Arguments nmono_in_leif [disp T A f C].
Arguments mono_leif [disp T f C].
Arguments nmono_leif [disp T f C].
Arguments min_idPl {disp T x y}.
Arguments max_idPr {disp T x y}.
Arguments comparable_min_idPr {disp T x y _}.
Arguments comparable_max_idPl {disp T x y _}.

Module Import DualPOrder.
Section DualPOrder.


Context {disp : unit}.
Variable T : porderType disp.

Lemma dual_lt_def (x y : T) : gt x y = (y != x) && ge x y.

Fact dual_le_anti : antisymmetric (@ge _ T).


Lemma leEdual (x y : T) : (x <=^d y :> T^d) = (y x).
Lemma ltEdual (x y : T) : (x <^d y :> T^d) = (y < x).

End DualPOrder.


End DualPOrder.

Module Import DualLattice.
Section DualLattice.
Context {disp : unit}.
Variable L : latticeType disp.
Implicit Types (x y : L).

Lemma meetC : commutative (@meet _ L).
Lemma joinC : commutative (@join _ L).

Lemma meetA : associative (@meet _ L).
Lemma joinA : associative (@join _ L).

Lemma joinKI y x : x `&` (x `|` y) = x.
Lemma meetKU y x : x `|` (x `&` y) = x.

Lemma joinKIC y x : x `&` (y `|` x) = x.
Lemma meetKUC y x : x `|` (y `&` x) = x.

Lemma meetUK x y : (x `&` y) `|` y = y.
Lemma joinIK x y : (x `|` y) `&` y = y.

Lemma meetUKC x y : (y `&` x) `|` y = y.
Lemma joinIKC x y : (y `|` x) `&` y = y.

Lemma leEmeet x y : (x y) = (x `&` y == x).

Lemma leEjoin x y : (x y) = (x `|` y == y).

Fact dual_leEmeet (x y : L^d) : (x y) = (x `|` y == x).


Lemma meetEdual x y : ((x : L^d) `&^d` y) = (x `|` y).
Lemma joinEdual x y : ((x : L^d) `|^d` y) = (x `&` y).

End DualLattice.
End DualLattice.

Module Import LatticeTheoryMeet.
Section LatticeTheoryMeet.
Context {disp : unit} {L : latticeType disp}.
Implicit Types (x y : L).

lattice theory
Lemma meetAC : right_commutative (@meet _ L).
Lemma meetCA : left_commutative (@meet _ L).
Lemma meetACA : interchange (@meet _ L) (@meet _ L).

Lemma meetxx x : x `&` x = x.

Lemma meetKI y x : x `&` (x `&` y) = x `&` y.
Lemma meetIK y x : (x `&` y) `&` y = x `&` y.
Lemma meetKIC y x : x `&` (y `&` x) = x `&` y.
Lemma meetIKC y x : y `&` x `&` y = x `&` y.

interaction with order

Lemma lexI x y z : (x y `&` z) = (x y) && (x z).

Lemma leIxl x y z : y x y `&` z x.

Lemma leIxr x y z : z x y `&` z x.

Lemma leIx2 x y z : (y x) || (z x) y `&` z x.

Lemma leIr x y : y `&` x x.

Lemma leIl x y : x `&` y x.

Lemma meet_idPl {x y} : reflect (x `&` y = x) (x y).
Lemma meet_idPr {x y} : reflect (y `&` x = x) (x y).

Lemma meet_l x y : x y x `&` y = x.
Lemma meet_r x y : y x x `&` y = y.

Lemma leIidl x y : (x x `&` y) = (x y).
Lemma leIidr x y : (x y `&` x) = (x y).

Lemma eq_meetl x y : (x `&` y == x) = (x y).

Lemma eq_meetr x y : (x `&` y == y) = (y x).

Lemma leI2 x y z t : x z y t x `&` y z `&` t.

End LatticeTheoryMeet.
End LatticeTheoryMeet.

Module Import LatticeTheoryJoin.
Section LatticeTheoryJoin.
Context {disp : unit} {L : latticeType disp}.
Implicit Types (x y : L).

lattice theory
Lemma joinAC : right_commutative (@join _ L).
Lemma joinCA : left_commutative (@join _ L).
Lemma joinACA : interchange (@join _ L) (@join _ L).

Lemma joinxx x : x `|` x = x.

Lemma joinKU y x : x `|` (x `|` y) = x `|` y.
Lemma joinUK y x : (x `|` y) `|` y = x `|` y.
Lemma joinKUC y x : x `|` (y `|` x) = x `|` y.
Lemma joinUKC y x : y `|` x `|` y = x `|` y.

interaction with order
Lemma leUx x y z : (x `|` y z) = (x z) && (y z).
Lemma lexUl x y z : x y x y `|` z.
Lemma lexUr x y z : x z x y `|` z.
Lemma lexU2 x y z : (x y) || (x z) x y `|` z.

Lemma leUr x y : x y `|` x.
Lemma leUl x y : x x `|` y.

Lemma join_idPr {x y} : reflect (x `|` y = y) (x y).
Lemma join_idPl {x y} : reflect (y `|` x = y) (x y).

Lemma join_l x y : y x x `|` y = x.
Lemma join_r x y : x y x `|` y = y.

Lemma leUidl x y : (x `|` y y) = (x y).
Lemma leUidr x y : (y `|` x y) = (x y).

Lemma eq_joinl x y : (x `|` y == x) = (y x).
Lemma eq_joinr x y : (x `|` y == y) = (x y).

Lemma leU2 x y z t : x z y t x `|` y z `|` t.

Lemma lcomparableP x y : incomparel x y
  (min y x) (min x y) (max y x) (max x y)
  (y `&` x) (x `&` y) (y `|` x) (x `|` y)
  (y == x) (x == y) (x y) (x y) (x > y) (x < y) (y >=< x) (x >=< y).

Lemma lcomparable_ltgtP x y : x >=< y
  comparel x y (min y x) (min x y) (max y x) (max x y)
               (y `&` x) (x `&` y) (y `|` x) (x `|` y)
               (y == x) (x == y) (x y) (x y) (x > y) (x < y).

Lemma lcomparable_leP x y : x >=< y
  lel_xor_gt x y (min y x) (min x y) (max y x) (max x y)
                 (y `&` x) (x `&` y) (y `|` x) (x `|` y) (x y) (y < x).

Lemma lcomparable_ltP x y : x >=< y
  ltl_xor_ge x y (min y x) (min x y) (max y x) (max x y)
                 (y `&` x) (x `&` y) (y `|` x) (x `|` y) (y x) (x < y).

End LatticeTheoryJoin.
End LatticeTheoryJoin.

Arguments meet_idPl {disp L x y}.
Arguments join_idPl {disp L x y}.

Module Import DistrLatticeTheory.
Section DistrLatticeTheory.
Context {disp : unit}.
Variable L : distrLatticeType disp.
Implicit Types (x y : L).

Lemma meetUl : left_distributive (@meet _ L) (@join _ L).

Lemma meetUr : right_distributive (@meet _ L) (@join _ L).

Lemma joinIl : left_distributive (@join _ L) (@meet _ L).

Lemma joinIr : right_distributive (@join _ L) (@meet _ L).


End DistrLatticeTheory.
End DistrLatticeTheory.

Module Import TotalTheory.
Section TotalTheory.
Context {disp : unit} {T : orderType disp}.
Implicit Types (x y z t : T) (s : seq T).

Definition le_total : total (<=%O : rel T) := le_total.
Hint Resolve le_total : core.

Lemma ge_total : total (>=%O : rel T).
Hint Resolve ge_total : core.

Lemma comparableT x y : x >=< y.
Hint Resolve comparableT : core.

Lemma sort_le_sorted s : sorted <=%O (sort <=%O s).
Hint Resolve sort_le_sorted : core.

Lemma sort_lt_sorted s : sorted <%O (sort <=%O s) = uniq s.

Lemma perm_sort_leP s1 s2 : reflect (sort <=%O s1 = sort <=%O s2) (perm_eq s1 s2).

Lemma filter_sort_le p s : filter p (sort <=%O s) = sort <=%O (filter p s).

Lemma mask_sort_le s (m : bitseq) :
  {m_s : bitseq | mask m_s (sort <=%O s) = sort <=%O (mask m s)}.

Lemma sorted_mask_sort_le s (m : bitseq) :
  sorted <=%O (mask m s) {m_s : bitseq | mask m_s (sort <=%O s) = mask m s}.

Lemma subseq_sort_le : {homo sort <=%O : s1 s2 / @subseq T s1 s2}.

Lemma sorted_subseq_sort_le s1 s2 :
  subseq s1 s2 sorted <=%O s1 subseq s1 (sort <=%O s2).

Lemma mem2_sort_le s x y : x y mem2 s x y mem2 (sort <=%O s) x y.

Lemma leNgt x y : (x y) = ~~ (y < x).

Lemma ltNge x y : (x < y) = ~~ (y x).

Definition ltgtP x y := LatticeTheoryJoin.lcomparable_ltgtP (comparableT x y).
Definition leP x y := LatticeTheoryJoin.lcomparable_leP (comparableT x y).
Definition ltP x y := LatticeTheoryJoin.lcomparable_ltP (comparableT x y).

Lemma wlog_le P :
     ( x y, P y x P x y) ( x y, x y P x y)
    x y, P x y.

Lemma wlog_lt P :
    ( x, P x x)
    ( x y, (P y x P x y)) ( x y, x < y P x y)
   x y, P x y.

Lemma neq_lt x y : (x != y) = (x < y) || (y < x).

Lemma lt_total x y : x != y (x < y) || (y < x).

Lemma eq_leLR x y z t :
  (x y z t) (y < x t < z) (x y) = (z t).

Lemma eq_leRL x y z t :
  (x y z t) (y < x t < z) (z t) = (x y).

Lemma eq_ltLR x y z t :
  (x < y z < t) (y x t z) (x < y) = (z < t).

Lemma eq_ltRL x y z t :
  (x < y z < t) (y x t z) (z < t) = (x < y).

max and min is join and meet

Lemma meetEtotal x y : x `&` y = min x y.
Lemma joinEtotal x y : x `|` y = max x y.

max and min theory

Lemma minEgt x y : min x y = if x > y then y else x.
Lemma maxEgt x y : max x y = if x > y then x else y.
Lemma minEge x y : min x y = if x y then y else x.
Lemma maxEge x y : max x y = if x y then x else y.

Lemma minC : commutative (min : T T T).

Lemma maxC : commutative (max : T T T).

Lemma minA : associative (min : T T T).

Lemma maxA : associative (max : T T T).

Lemma minAC : right_commutative (min : T T T).

Lemma maxAC : right_commutative (max : T T T).

Lemma minCA : left_commutative (min : T T T).

Lemma maxCA : left_commutative (max : T T T).

Lemma minACA : interchange (min : T T T) min.

Lemma maxACA : interchange (max : T T T) max.

Lemma eq_minr x y : (min x y == y) = (y x).

Lemma eq_maxl x y : (max x y == x) = (y x).

Lemma min_idPr x y : reflect (min x y = y) (y x).

Lemma max_idPl x y : reflect (max x y = x) (y x).

Lemma le_min z x y : (z min x y) = (z x) && (z y).

Lemma ge_min z x y : (min x y z) = (x z) || (y z).

Lemma lt_min z x y : (z < min x y) = (z < x) && (z < y).

Lemma gt_min z x y : (min x y < z) = (x < z) || (y < z).

Lemma le_max z x y : (z max x y) = (z x) || (z y).

Lemma ge_max z x y : (max x y z) = (x z) && (y z).

Lemma lt_max z x y : (z < max x y) = (z < x) || (z < y).

Lemma gt_max z x y : (max x y < z) = (x < z) && (y < z).

Lemma minxK x y : max (min x y) y = y.
Lemma minKx x y : max x (min x y) = x.
Lemma maxxK x y : min (max x y) y = y.
Lemma maxKx x y : min x (max x y) = x.

Lemma max_minl : left_distributive (max : T T T) min.

Lemma min_maxl : left_distributive (min : T T T) max.

Lemma max_minr : right_distributive (max : T T T) min.

Lemma min_maxr : right_distributive (min : T T T) max.


Lemma leIx x y z : (meet y z x) = (y x) || (z x).

Lemma lexU x y z : (x join y z) = (x y) || (x z).

Lemma ltxI x y z : (x < meet y z) = (x < y) && (x < z).

Lemma ltIx x y z : (meet y z < x) = (y < x) || (z < x).

Lemma ltxU x y z : (x < join y z) = (x < y) || (x < z).

Lemma ltUx x y z : (join y z < x) = (y < x) && (z < x).

Definition ltexI := (@lexI _ T, ltxI).
Definition lteIx := (leIx, ltIx).
Definition ltexU := (lexU, ltxU).
Definition lteUx := (@leUx _ T, ltUx).

lteif

Lemma lteifNE x y C : x < y ?<= if ~~ C = ~~ (y < x ?<= if C).

Lemma lteif_minr z x y C :
  (z < Order.min x y ?<= if C) = (z < x ?<= if C) && (z < y ?<= if C).

Lemma lteif_minl z x y C :
  (Order.min x y < z ?<= if C) = (x < z ?<= if C) || (y < z ?<= if C).

Lemma lteif_maxr z x y C :
  (z < Order.max x y ?<= if C) = (z < x ?<= if C) || (z < y ?<= if C).

Lemma lteif_maxl z x y C :
  (Order.max x y < z ?<= if C) = (x < z ?<= if C) && (y < z ?<= if C).

Section ArgExtremum.

Context (I : finType) (i0 : I) (P : {pred I}) (F : I T) (Pi0 : P i0).

Lemma arg_minP: extremum_spec <=%O P F (arg_min i0 P F).

Lemma arg_maxP: extremum_spec >=%O P F (arg_max i0 P F).

End ArgExtremum.

Lemma count_le_gt x s : count ( x) s = size s - count (> x) s.

Lemma count_lt_ge x s : count (< x) s = size s - count ( x) s.

Section bigminmax_Type.
Variables (I : Type) (r : seq I) (x : T).
Implicit Types (P : pred I) (F : I T).

Lemma bigmin_mkcond P F : \big[min/x]_(i <- r | P i) F i =
  \big[min/x]_(i <- r) (if P i then F i else x).

Lemma bigmax_mkcond P F :
  \big[max/x]_(i <- r | P i) F i = \big[max/x]_(i <- r) if P i then F i else x.

Lemma bigmin_mkcondl P Q F :
  \big[min/x]_(i <- r | P i && Q i) F i
  = \big[min/x]_(i <- r | Q i) if P i then F i else x.

Lemma bigmin_mkcondr P Q F :
  \big[min/x]_(i <- r | P i && Q i) F i
  = \big[min/x]_(i <- r | P i) if Q i then F i else x.

Lemma bigmax_mkcondl P Q F :
  \big[max/x]_(i <- r | P i && Q i) F i
  = \big[max/x]_(i <- r | Q i) if P i then F i else x.

Lemma bigmax_mkcondr P Q F :
  \big[max/x]_(i <- r | P i && Q i) F i
  = \big[max/x]_(i <- r | P i) if Q i then F i else x.

Lemma bigmin_split P F1 F2 :
  \big[min/x]_(i <- r | P i) (min (F1 i) (F2 i)) =
    min (\big[min/x]_(i <- r | P i) F1 i) (\big[min/x]_(i <- r | P i) F2 i).

Lemma bigmax_split P F1 F2 :
  \big[max/x]_(i <- r | P i) (max (F1 i) (F2 i)) =
    max (\big[max/x]_(i <- r | P i) F1 i) (\big[max/x]_(i <- r | P i) F2 i).

Lemma bigmin_idl P F :
  \big[min/x]_(i <- r | P i) F i = min x (\big[min/x]_(i <- r | P i) F i).

Lemma bigmax_idl P F :
  \big[max/x]_(i <- r | P i) F i = max x (\big[max/x]_(i <- r | P i) F i).

Lemma bigmin_idr P F :
  \big[min/x]_(i <- r | P i) F i = min (\big[min/x]_(i <- r | P i) F i) x.

Lemma bigmax_idr P F :
  \big[max/x]_(i <- r | P i) F i = max (\big[max/x]_(i <- r | P i) F i) x.

Lemma bigminID a P F : \big[min/x]_(i <- r | P i) F i =
  min (\big[min/x]_(i <- r | P i && a i) F i)
      (\big[min/x]_(i <- r | P i && ~~ a i) F i).

Lemma bigmaxID a P F : \big[max/x]_(i <- r | P i) F i =
  max (\big[max/x]_(i <- r | P i && a i) F i)
      (\big[max/x]_(i <- r | P i && ~~ a i) F i).

End bigminmax_Type.

Let ge_min_id (x y : T) : x min x y.
Let le_max_id (x y : T) : x max x y.

Lemma sub_bigmin [x0] I r (P P' : {pred I}) (F : I T) :
    ( i, P' i P i)
  \big[min/x0]_(i <- r | P i) F i \big[min/x0]_(i <- r | P' i) F i.

Lemma sub_bigmax [x0] I r (P P' : {pred I}) (F : I T) :
    ( i, P i P' i)
  \big[max/x0]_(i <- r | P i) F i \big[max/x0]_(i <- r | P' i) F i.

Lemma sub_bigmin_seq [x0] (I : eqType) r r' P (F : I T) : {subset r' r}
  \big[min/x0]_(i <- r | P i) F i \big[min/x0]_(i <- r' | P i) F i.

Lemma sub_bigmax_seq [x0] (I : eqType) r r' P (F : I T) : {subset r r'}
  \big[max/x0]_(i <- r | P i) F i \big[max/x0]_(i <- r' | P i) F i.

Lemma sub_bigmin_cond [x0] (I : eqType) r r' P P' (F : I T) :
    {subset [seq i <- r | P i] [seq i <- r' | P' i]}
  \big[min/x0]_(i <- r' | P' i) F i \big[min/x0]_(i <- r | P i) F i.

Lemma sub_bigmax_cond [x0] (I : eqType) r r' P P' (F : I T) :
    {subset [seq i <- r | P i] [seq i <- r' | P' i]}
  \big[max/x0]_(i <- r | P i) F i \big[max/x0]_(i <- r' | P' i) F i.

Lemma sub_in_bigmin [x0] [I : eqType] (r : seq I) (P P' : {pred I}) F :
    {in r, i, P' i P i}
  \big[min/x0]_(i <- r | P i) F i \big[min/x0]_(i <- r | P' i) F i.

Lemma sub_in_bigmax [x0] [I : eqType] (r : seq I) (P P' : {pred I}) F :
    {in r, i, P i P' i}
  \big[max/x0]_(i <- r | P i) F i \big[max/x0]_(i <- r | P' i) F i.

Lemma le_bigmin_nat [x0] n m n' m' P (F : nat T) :
    (n n')%N (m' m)%N
  \big[min/x0]_(n i < m | P i) F i \big[min/x0]_(n' i < m' | P i) F i.

Lemma le_bigmax_nat [x0] n m n' m' P (F : nat T) :
    (n' n)%N (m m')%N
  \big[max/x0]_(n i < m | P i) F i \big[max/x0]_(n' i < m' | P i) F i.

Lemma le_bigmin_nat_cond [x0] n m n' m' (P P' : pred nat) (F : nat T) :
    (n n')%N (m' m)%N ( i, (n' i < m')%N P' i P i)
  \big[min/x0]_(n i < m | P i) F i \big[min/x0]_(n' i < m' | P' i) F i.

Lemma le_bigmax_nat_cond [x0] n m n' m' (P P' : {pred nat}) (F : nat T) :
    (n' n)%N (m m')%N ( i, (n i < m)%N P i P' i)
  \big[max/x0]_(n i < m | P i) F i \big[max/x0]_(n' i < m' | P' i) F i.

Lemma le_bigmin_ord [x0] n m (P : pred nat) (F : nat T) : (m n)%N
  \big[min/x0]_(i < n | P i) F i \big[min/x0]_(i < m | P i) F i.

Lemma le_bigmax_ord [x0] n m (P : {pred nat}) (F : nat T) : (n m)%N
  \big[max/x0]_(i < n | P i) F i \big[max/x0]_(i < m | P i) F i.

Lemma le_bigmin_ord_cond [x0] n m (P P' : pred nat) (F : nat T) :
    (m n)%N ( i : 'I_m, P' i P i)
  \big[min/x0]_(i < n | P i) F i \big[min/x0]_(i < m | P' i) F i.

Lemma le_bigmax_ord_cond [x0] n m (P P' : {pred nat}) (F : nat T) :
    (n m)%N ( i : 'I_n, P i P' i)
  \big[max/x0]_(i < n | P i) F i \big[max/x0]_(i < m | P' i) F i.

Lemma subset_bigmin [x0] [I : finType] [A A' P : {pred I}] (F : I T) :
    A' \subset A
  \big[min/x0]_(i in A | P i) F i \big[min/x0]_(i in A' | P i) F i.

Lemma subset_bigmax [x0] [I : finType] (A A' P : {pred I}) (F : I T) :
    A \subset A'
  \big[max/x0]_(i in A | P i) F i \big[max/x0]_(i in A' | P i) F i.

Lemma subset_bigmin_cond [x0] (I : finType) (A A' P P' : {pred I}) (F : I T) :
    [set i in A' | P' i] \subset [set i in A | P i]
  \big[min/x0]_(i in A | P i) F i \big[min/x0]_(i in A' | P' i) F i.

Lemma subset_bigmax_cond [x0] (I : finType) (A A' P P' : {pred I}) (F : I T) :
    [set i in A | P i] \subset [set i in A' | P' i]
  \big[max/x0]_(i in A | P i) F i \big[max/x0]_(i in A' | P' i) F i.

Section bigminmax_eqType.
Variable (I : eqType) (r : seq I) (x : T).
Implicit Types (P : pred I) (F : I T).

Lemma bigmin_le_id P F : \big[min/x]_(i <- r | P i) F i x.

Lemma bigmax_ge_id P F : \big[max/x]_(i <- r | P i) F i x.

Lemma bigmin_eq_id P F :
  ( i, P i x F i) \big[min/x]_(i <- r | P i) F i = x.

Lemma bigmax_eq_id P F :
  ( i, P i x F i) \big[max/x]_(i <- r | P i) F i = x.

End bigminmax_eqType.

Section bigminmax_finType.
Variable (I : finType) (x : T).
Implicit Types (P : pred I) (F : I T).

Lemma bigminD1 j P F : P j
  \big[min/x]_(i | P i) F i = min (F j) (\big[min/x]_(i | P i && (i != j)) F i).

Lemma bigmaxD1 j P F : P j
  \big[max/x]_(i | P i) F i = max (F j) (\big[max/x]_(i | P i && (i != j)) F i).

Lemma bigmin_le_cond j P F : P j \big[min/x]_(i | P i) F i F j.

Lemma le_bigmax_cond j P F : P j F j \big[max/x]_(i | P i) F i.

Lemma bigmin_le j F : \big[min/x]_i F i F j.

Lemma le_bigmax F j : F j \big[max/x]_i F i.

Lemma bigmin_inf j P m F : P j F j m \big[min/x]_(i | P i) F i m.

NB: as of [2022-08-02], bigop.bigmax_sup already exists for nat
Lemma bigmax_sup j P m F : P j m F j m \big[max/x]_(i | P i) F i.

Lemma bigmin_geP m P F :
  reflect (m x i, P i m F i)
          (m \big[min/x]_(i | P i) F i).

Lemma bigmax_leP m P F :
  reflect (x m i, P i F i m)
          (\big[max/x]_(i | P i) F i m).

Lemma bigmin_gtP m P F :
  reflect (m < x i, P i m < F i) (m < \big[min/x]_(i | P i) F i).

Lemma bigmax_ltP m P F :
  reflect (x < m i, P i F i < m) (\big[max/x]_(i | P i) F i < m).

Lemma bigmin_eq_arg j P F : P j ( i, P i F i x)
  \big[min/x]_(i | P i) F i = F [arg min_(i < j | P i) F i].

Lemma bigmax_eq_arg j P F : P j ( i, P i x F i)
  \big[max/x]_(i | P i) F i = F [arg max_(i > j | P i) F i].

Lemma eq_bigmin j P F : P j ( i, P i F i x)
  {i0 | i0 \in P & \big[min/x]_(i | P i) F i = F i0}.

Lemma eq_bigmax j P F : P j ( i, P i x F i)
  {i0 | i0 \in P & \big[max/x]_(i | P i) F i = F i0}.

Lemma le_bigmin2 P F1 F2 : ( i, P i F1 i F2 i)
  \big[min/x]_(i | P i) F1 i \big[min/x]_(i | P i) F2 i.

Lemma le_bigmax2 P F1 F2 : ( i, P i F1 i F2 i)
  \big[max/x]_(i | P i) F1 i \big[max/x]_(i | P i) F2 i.

Lemma bigmaxUl (A B : {set I}) F :
  \big[max/x]_(i in A) F i \big[max/x]_(i in A :|: B) F i.

Lemma bigmaxUr (A B : {set I}) F :
  \big[max/x]_(i in B) F i \big[max/x]_(i in A :|: B) F i.

Lemma bigminUl (A B : {set I}) F :
  \big[min/x]_(i in A) F i \big[min/x]_(i in A :|: B) F i.

Lemma bigminUr (A B : {set I}) F :
  \big[min/x]_(i in B) F i \big[min/x]_(i in A :|: B) F i.

Lemma bigmaxIl (A B : {set I}) F :
  \big[max/x]_(i in A) F i \big[max/x]_(i in A :&: B) F i.

Lemma bigmaxIr (A B : {set I}) F :
  \big[max/x]_(i in B) F i \big[max/x]_(i in A :&: B) F i.

Lemma bigminIl (A B : {set I}) F :
  \big[min/x]_(i in A) F i \big[min/x]_(i in A :&: B) F i.

Lemma bigminIr (A B : {set I}) F :
  \big[min/x]_(i in B) F i \big[min/x]_(i in A :&: B) F i.

Lemma bigmaxD (A B : {set I}) F :
  \big[max/x]_(i in B) F i \big[max/x]_(i in B :\: A) F i.

Lemma bigminD (A B : {set I}) F :
  \big[min/x]_(i in B) F i \big[min/x]_(i in B :\: A) F i.

Lemma bigmaxU (A B : {set I}) F :
  \big[max/x]_(i in A :|: B) F i
  = max (\big[max/x]_(i in A) F i) (\big[max/x]_(i in B) F i).

Lemma bigminU (A B : {set I}) F :
  \big[min/x]_(i in A :|: B) F i
  = min (\big[min/x]_(i in A) F i) (\big[min/x]_(i in B) F i).

Lemma bigmin_set1 j F : \big[min/x]_(i in [set j]) F i = min (F j) x.

Lemma bigmax_set1 j F : \big[max/x]_(i in [set j]) F i = max (F j) x.

End bigminmax_finType.

Lemma bigmin_imset [I J : finType] x [h : I J] [A : {set I}] (F : J T) :
  \big[min/x]_(j in [set h x | x in A]) F j = \big[min/x]_(i in A) F (h i).

Lemma bigmax_imset [I J : finType] x [h : I J] [A : {set I}] (F : J T) :
  \big[max/x]_(j in [set h x | x in A]) F j = \big[max/x]_(i in A) F (h i).

End TotalTheory.

#[global] Hint Resolve le_total : core.
#[global] Hint Resolve ge_total : core.
#[global] Hint Resolve comparableT : core.
#[global] Hint Resolve sort_le_sorted : core.

Arguments min_idPr {disp T x y}.
Arguments max_idPl {disp T x y}.
Arguments bigmin_mkcond {disp T I r}.
Arguments bigmax_mkcond {disp T I r}.
Arguments bigminID {disp T I r}.
Arguments bigmaxID {disp T I r}.
Arguments bigminD1 {disp T I x} j.
Arguments bigmaxD1 {disp T I x} j.
Arguments bigmin_inf {disp T I x} j.
Arguments bigmax_sup {disp T I x} j.
Arguments bigmin_eq_arg {disp T I} x j.
Arguments bigmax_eq_arg {disp T I} x j.
Arguments eq_bigmin {disp T I x} j.
Arguments eq_bigmax {disp T I x} j.

contra lemmas

Section ContraTheory.
Context {disp1 disp2 : unit} {T1 : porderType disp1} {T2 : orderType disp2}.
Implicit Types (x y : T1) (z t : T2) (b : bool) (m n : nat) (P : Prop).

Lemma contraTle b z t : (t < z ~~ b) (b z t).

Lemma contraTlt b z t : (t z ~~ b) (b z < t).

Lemma contraPle P z t : (t < z ¬ P) (P z t).

Lemma contraPlt P z t : (t z ¬ P) (P z < t).

Lemma contraNle b z t : (t < z b) (~~ b z t).

Lemma contraNlt b z t : (t z b) (~~ b z < t).

Lemma contra_not_le P z t : (t < z P) (¬ P z t).

Lemma contra_not_lt P z t : (t z P) (¬ P z < t).

Lemma contraFle b z t : (t < z b) (b = false z t).

Lemma contraFlt b z t : (t z b) (b = false z < t).

Lemma contra_leq_le m n z t : (t < z (n < m)%N) ((m n)%N z t).

Lemma contra_leq_lt m n z t : (t z (n < m)%N) ((m n)%N z < t).

Lemma contra_ltn_le m n z t : (t < z (n m)%N) ((m < n)%N z t).

Lemma contra_ltn_lt m n z t : (t z (n m)%N) ((m < n)%N z < t).

Lemma contra_le x y z t : (t < z y < x) (x y z t).

Lemma contra_le_lt x y z t : (t z y < x) (x y z < t).

Lemma contra_lt_le x y z t : (t < z y x) (x < y z t).

Lemma contra_lt x y z t : (t z y x) (x < y z < t).

End ContraTheory.

Section TotalMonotonyTheory.

Context {disp : unit} {disp' : unit}.
Context {T : orderType disp} {T' : porderType disp'}.
Variables (D : {pred T}) (f : T T').
Implicit Types (x y z : T) (u v w : T').

Let leT_anti := @le_anti _ T.
Let leT'_anti := @le_anti _ T'.
Let ltT_neqAle := @lt_neqAle _ T.
Let ltT'_neqAle := @lt_neqAle _ T'.
Let ltT_def := @lt_def _ T.
Let leT_total := @le_total _ T.

Lemma le_mono : {homo f : x y / x < y} {mono f : x y / x y}.

Lemma le_nmono : {homo f : x y /~ x < y} {mono f : x y /~ x y}.

Lemma le_mono_in :
  {in D &, {homo f : x y / x < y}} {in D &, {mono f : x y / x y}}.

Lemma le_nmono_in :
  {in D &, {homo f : x y /~ x < y}} {in D &, {mono f : x y /~ x y}}.

End TotalMonotonyTheory.

#[deprecated(since="mathcomp 2.1.0", note="Use comparable_le_min instead.")]
Notation comparable_le_minr := comparable_le_min.
#[deprecated(since="mathcomp 2.1.0", note="Use comparable_ge_min instead.")]
Notation comparable_le_minl := comparable_ge_min.
#[deprecated(since="mathcomp 2.1.0", note="Use comparable_gt_min instead.")]
Notation comparable_lt_minl := comparable_gt_min.
#[deprecated(since="mathcomp 2.1.0", note="Use comparable_lt_min instead.")]
Notation comparable_lt_minr := comparable_lt_min.
#[deprecated(since="mathcomp 2.1.0", note="Use comparable_le_max instead.")]
Notation comparable_le_maxr := comparable_le_max.
#[deprecated(since="mathcomp 2.1.0", note="Use comparable_ge_max instead.")]
Notation comparable_le_maxl := comparable_ge_max.
#[deprecated(since="mathcomp 2.1.0", note="Use comparable_lt_max instead.")]
Notation comparable_lt_maxr := comparable_lt_max.
#[deprecated(since="mathcomp 2.1.0", note="Use comparable_gt_max instead.")]
Notation comparable_lt_maxl := comparable_gt_max.
#[deprecated(since="mathcomp 2.1.0", note="Use ge_max instead.")]
Notation le_maxl := ge_max.
#[deprecated(since="mathcomp 2.1.0", note="Use le_max instead.")]
Notation le_maxr := le_max.
#[deprecated(since="mathcomp 2.1.0", note="Use gt_max instead.")]
Notation lt_maxl := gt_max.
#[deprecated(since="mathcomp 2.1.0", note="Use lt_max instead.")]
Notation lt_maxr := lt_max.
#[deprecated(since="mathcomp 2.1.0", note="Use lt_min instead.")]
Notation lt_minr := lt_min.
#[deprecated(since="mathcomp 2.1.0", note="Use gt_max instead.")]
Notation lt_minl := gt_min.
#[deprecated(since="mathcomp 2.1.0", note="Use le_min instead.")]
Notation le_minr := le_min.
#[deprecated(since="mathcomp 2.1.0", note="Use ge_min instead.")]
Notation le_minl := ge_min.

End TotalTheory.

Module Import BLatticeTheory.
Section BLatticeTheory.
Context {disp : unit} {L : bLatticeType disp}.
Implicit Types (I : finType) (T : eqType) (x y z : L).

Non-distributive lattice theory with \bot & \top
Lemma le0x x : \bot x.
Hint Resolve le0x : core.

Lemma lex0 x : (x \bot) = (x == \bot).

Lemma ltx0 x : (x < \bot) = false.

Lemma lt0x x : (\bot < x) = (x != \bot).

Lemma meet0x : left_zero \bot (@meet _ L).

Lemma meetx0 : right_zero \bot (@meet _ L).

Lemma join0x : left_id \bot (@join _ L).

Lemma joinx0 : right_id \bot (@join _ L).

Lemma join_eq0 x y : (x `|` y == \bot) = (x == \bot) && (y == \bot).

Variant eq0_xor_gt0 x : bool bool Set :=
    Eq0NotPOs : x = \bot eq0_xor_gt0 x true false
  | POsNotEq0 : \bot < x eq0_xor_gt0 x false true.

Lemma posxP x : eq0_xor_gt0 x (x == \bot) (\bot < x).


Lemma joins_sup_seq T (r : seq T) (P : {pred T}) (F : T L) (x : T) :
  x \in r P x F x \join_(i <- r | P i) F i.

Lemma joins_min_seq T (r : seq T) (P : {pred T}) (F : T L) (x : T) (l : L) :
  x \in r P x l F x l \join_(x <- r | P x) F x.

Lemma joins_sup I (j : I) (P : {pred I}) (F : I L) :
  P j F j \join_(i | P i) F i.

Lemma joins_min I (j : I) (l : L) (P : {pred I}) (F : I L) :
  P j l F j l \join_(i | P i) F i.

Lemma joins_le J (r : seq J) (P : {pred J}) (F : J L) (u : L) :
  ( x : J, P x F x u) \join_(x <- r | P x) F x u.

Lemma joinsP_seq T (r : seq T) (P : {pred T}) (F : T L) (u : L) :
  reflect ( x : T, x \in r P x F x u)
          (\join_(x <- r | P x) F x u).

Lemma joinsP I (u : L) (P : {pred I}) (F : I L) :
  reflect ( i : I, P i F i u) (\join_(i | P i) F i u).

Lemma le_joins I (A B : {set I}) (F : I L) :
  A \subset B \join_(i in A) F i \join_(i in B) F i.

Lemma joins_setU I (A B : {set I}) (F : I L) :
  \join_(i in (A :|: B)) F i = \join_(i in A) F i `|` \join_(i in B) F i.

Lemma joins_seq I (r : seq I) (F : I L) :
  \join_(i <- r) F i = \join_(i in r) F i.

End BLatticeTheory.

End BLatticeTheory.

Module Import DualTBLattice.
Section DualTBLattice.
Context {disp : unit} {L : tbLatticeType disp}.

FIXME: BUG? HB.instance Definition _ := TBLattice.on L^d.

Lemma botEdual : (dual_bottom : L^d) = \top :> L.
Lemma topEdual : (dual_top : L^d) = \bot :> L.

End DualTBLattice.


End DualTBLattice.

Module Import TLatticeTheory.
Section TLatticeTheory.
Context {disp : unit} {L : tLatticeType disp}.
Implicit Types (I : finType) (T : eqType) (x y : L).


Lemma lex1 (x : L) : x top.

Hint Resolve lex1 : core.

Lemma meetx1 : right_id \top (@meet _ L).

Lemma meet1x : left_id \top (@meet _ L).

Lemma joinx1 : right_zero \top (@join _ L).

Lemma join1x : left_zero \top (@join _ L).

Lemma le1x x : (\top x) = (x == \top).

Lemma meet_eq1 x y : (x `&` y == \top) = (x == \top) && (y == \top).



Lemma meets_inf_seq T (r : seq T) (P : {pred T}) (F : T L) (x : T) :
  x \in r P x \meet_(i <- r | P i) F i F x.

Lemma meets_max_seq T (r : seq T) (P : {pred T}) (F : T L) (x : T) (u : L) :
  x \in r P x F x u \meet_(x <- r | P x) F x u.

Lemma meets_inf I (j : I) (P : {pred I}) (F : I L) :
   P j \meet_(i | P i) F i F j.

Lemma meets_max I (j : I) (u : L) (P : {pred I}) (F : I L) :
   P j F j u \meet_(i | P i) F i u.

Lemma meets_ge J (r : seq J) (P : {pred J}) (F : J L) (u : L) :
  ( x : J, P x u F x) u \meet_(x <- r | P x) F x.

Lemma meetsP_seq T (r : seq T) (P : {pred T}) (F : T L) (l : L) :
  reflect ( x : T, x \in r P x l F x)
          (l \meet_(x <- r | P x) F x).

Lemma meetsP I (l : L) (P : {pred I}) (F : I L) :
   reflect ( i : I, P i l F i) (l \meet_(i | P i) F i).

Lemma le_meets I (A B : {set I}) (F : I L) :
   A \subset B \meet_(i in B) F i \meet_(i in A) F i.

Lemma meets_setU I (A B : {set I}) (F : I L) :
   \meet_(i in (A :|: B)) F i = \meet_(i in A) F i `&` \meet_(i in B) F i.

Lemma meets_seq I (r : seq I) (F : I L) :
   \meet_(i <- r) F i = \meet_(i in r) F i.

End TLatticeTheory.

End TLatticeTheory.

Module Import TBLatticeTheory.
Section TBLatticeTheory.
Context {disp : unit} {L : tbLatticeType disp}.



End TBLatticeTheory.

End TBLatticeTheory.

Module Import BDistrLatticeTheory.
Section BDistrLatticeTheory.
Context {disp : unit} {L : bDistrLatticeType disp}.
Implicit Types (I : finType) (T : eqType) (x y z : L).
Distributive lattice theory with \bot & \top

Lemma leU2l_le y t x z : x `&` t = \bot x `|` y z `|` t x z.

Lemma leU2r_le y t x z : x `&` t = \bot y `|` x t `|` z x z.

Lemma disjoint_lexUl z x y : x `&` z = \bot (x y `|` z) = (x y).

Lemma disjoint_lexUr z x y : x `&` z = \bot (x z `|` y) = (x y).

Lemma leU2E x y z t : x `&` t = \bot y `&` z = \bot
  (x `|` y z `|` t) = (x z) && (y t).

Lemma joins_disjoint I (d : L) (P : {pred I}) (F : I L) :
   ( i : I, P i d `&` F i = \bot) d `&` \join_(i | P i) F i = \bot.

End BDistrLatticeTheory.
End BDistrLatticeTheory.

Module Import DualTBDistrLattice.
Section DualTBDistrLattice.
Context {disp : unit} {L : tbDistrLatticeType disp}.


End DualTBDistrLattice.


End DualTBDistrLattice.

Module Import TBDistrLatticeTheory.
Section TBDistrLatticeTheory.
Context {disp : unit} {L : tbDistrLatticeType disp}.
Implicit Types (I : finType) (T : eqType) (x y : L).


Lemma leI2l_le y t x z : y `|` z = \top x `&` y z `&` t x z.

Lemma leI2r_le y t x z : y `|` z = \top y `&` x t `&` z x z.

Lemma cover_leIxl z x y : z `|` y = \top (x `&` z y) = (x y).

Lemma cover_leIxr z x y : z `|` y = \top (z `&` x y) = (x y).

Lemma leI2E x y z t : x `|` t = \top y `|` z = \top
  (x `&` y z `&` t) = (x z) && (y t).


Lemma meets_total I (d : L) (P : {pred I}) (F : I L) :
   ( i : I, P i d `|` F i = \top) d `|` \meet_(i | P i) F i = \top.

End TBDistrLatticeTheory.
End TBDistrLatticeTheory.

Module Import CBDistrLatticeTheory.
Section CBDistrLatticeTheory.
Context {disp : unit} {L : cbDistrLatticeType disp}.
Implicit Types (x y z : L).

Lemma diffKI x y : y `&` (x `\` y) = \bot.

Lemma diffIK x y : (x `\` y) `&` y = \bot.
#[deprecated(since="mathcomp 2.0.0", note="Use diffIK instead.")]
Notation subIK := diffIK.

Lemma meetIB z x y : (z `&` y) `&` (x `\` y) = \bot.

Lemma meetBI z x y : (x `\` y) `&` (z `&` y) = \bot.

Lemma joinIB y x : (x `&` y) `|` (x `\` y) = x.

Lemma joinBI y x : (x `\` y) `|` (x `&` y) = x.

Lemma joinIBC y x : (y `&` x) `|` (x `\` y) = x.

Lemma joinBIC y x : (x `\` y) `|` (y `&` x) = x.

Lemma leBx x y : x `\` y x.
Hint Resolve leBx : core.

Lemma diffxx x : x `\` x = \bot.
#[deprecated(since="mathcomp 2.0.0", note="Use diffxx instead.")]
Notation subxx := diffxx.

Lemma leBl z x y : x y x `\` z y `\` z.

Lemma diffKU y x : y `|` (x `\` y) = y `|` x.
#[deprecated(since="mathcomp 2.0.0", note="Use diffKU instead.")]
Notation subKU := diffKU.

Lemma diffUK y x : (x `\` y) `|` y = x `|` y.
#[deprecated(since="mathcomp 2.0.0", note="Use diffUK instead.")]
Notation subUK := diffUK.

Lemma leBKU y x : y x y `|` (x `\` y) = x.

Lemma leBUK y x : y x (x `\` y) `|` y = x.

Lemma leBLR x y z : (x `\` y z) = (x y `|` z).

Lemma diffUx x y z : (x `|` y) `\` z = (x `\` z) `|` (y `\` z).
#[deprecated(since="mathcomp 2.0.0", note="Use diffUx instead.")]
Notation subUx := diffUx.

Lemma diff_eq0 x y : (x `\` y == \bot) = (x y).
#[deprecated(since="mathcomp 2.0.0", note="Use diff_eq0 instead.")]
Notation sub_eq0 := diff_eq0.

Lemma joinxB x y z : x `|` (y `\` z) = ((x `|` y) `\` z) `|` (x `&` z).

Lemma joinBx x y z : (y `\` z) `|` x = ((y `|` x) `\` z) `|` (z `&` x).

Lemma leBr z x y : x y z `\` y z `\` x.

Lemma leB2 x y z t : x z t y x `\` y z `\` t.

Lemma meet_eq0E_diff z x y : x z (x `&` y == \bot) = (x z `\` y).
#[deprecated(since="mathcomp 2.0.0", note="Use meet_eq0E_sub instead.")]
Notation meet_eq0E_sub := meet_eq0E_diff.

Lemma leBRL x y z : (x z `\` y) = (x z) && (x `&` y == \bot).

Lemma eq_diff x y z : (x `\` y == z) = (z x y `|` z) && (z `&` y == \bot).
#[deprecated(since="mathcomp 2.0.0", note="Use eq_sub instead.")]
Notation eq_sub := eq_diff.

Lemma diffxU x y z : z `\` (x `|` y) = (z `\` x) `&` (z `\` y).
#[deprecated(since="mathcomp 2.0.0", note="Use diffxU instead.")]
Notation subxU := diffxU.

Lemma diffx0 x : x `\` \bot = x.
#[deprecated(since="mathcomp 2.0.0", note="Use diffx0 instead.")]
Notation subx0 := diffx0.

Lemma diff0x x : \bot `\` x = \bot.
#[deprecated(since="mathcomp 2.0.0", note="Use diff0x instead.")]
Notation sub0x := diff0x.

Lemma diffIx x y z : (x `&` y) `\` z = (x `\` z) `&` (y `\` z).
#[deprecated(since="mathcomp 2.0.0", note="Use diffIx instead.")]
Notation subIx := diffIx.

Lemma meetxB x y z : x `&` (y `\` z) = (x `&` y) `\` z.

Lemma meetBx x y z : (x `\` y) `&` z = (x `&` z) `\` y.

Lemma diffxI x y z : x `\` (y `&` z) = (x `\` y) `|` (x `\` z).
#[deprecated(since="mathcomp 2.0.0", note="Use diffxI instead.")]
Notation subxI := diffxI.

Lemma diffBx x y z : (x `\` y) `\` z = x `\` (y `|` z).
#[deprecated(since="mathcomp 2.0.0", note="Use diffBx instead.")]
Notation subBx := diffBx.

Lemma diffxB x y z : x `\` (y `\` z) = (x `\` y) `|` (x `&` z).
#[deprecated(since="mathcomp 2.0.0", note="Use diffxB instead.")]
Notation subxB := diffxB.

Lemma joinBK x y : (y `|` x) `\` x = (y `\` x).

Lemma joinBKC x y : (x `|` y) `\` x = (y `\` x).

Lemma disj_le x y : x `&` y == \bot x y = (x == \bot).

Lemma disj_leC x y : y `&` x == \bot x y = (x == \bot).

Lemma disj_diffl x y : x `&` y == \bot x `\` y = x.
#[deprecated(since="mathcomp 2.0.0", note="Use disj_diffl instead.")]
Notation disj_subl := disj_diffl.

Lemma disj_diffr x y : x `&` y == \bot y `\` x = y.
#[deprecated(since="mathcomp 2.0.0", note="Use disj_diffr instead.")]
Notation disj_subr := disj_diffr.

Lemma lt0B x y : x < y \bot < y `\` x.

End CBDistrLatticeTheory.
End CBDistrLatticeTheory.

Module Import CTBDistrLatticeTheory.
Section CTBDistrLatticeTheory.
Context {disp : unit} {L : ctbDistrLatticeType disp}.
Implicit Types (x y z : L).

Lemma complE x : ~` x = \top `\` x.

Lemma diff1x x : \top `\` x = ~` x.
#[deprecated(since="mathcomp 2.0.0", note="Use diff1x instead.")]
Notation sub1x := diff1x.

Lemma diffE x y : x `\` y = x `&` ~` y.
#[deprecated(since="mathcomp 2.0.0", note="Use diffE instead.")]
Notation subE := diffE.

Lemma complK : involutive (@compl _ L).

Lemma compl_inj : injective (@compl _ L).

Lemma disj_leC x y : (x `&` y == \bot) = (x ~` y).

Lemma leC x y : (~` x ~` y) = (y x).

Lemma complU x y : ~` (x `|` y) = ~` x `&` ~` y.

Lemma complI x y : ~` (x `&` y) = ~` x `|` ~` y.

Lemma joinxC x : x `|` ~` x = \top.

Lemma joinCx x : ~` x `|` x = \top.

Lemma meetxC x : x `&` ~` x = \bot.

Lemma meetCx x : ~` x `&` x = \bot.

Lemma compl1 : ~` \top = \bot :> L.

Lemma compl0 : ~` \bot = \top :> L.

Lemma complB x y : ~` (x `\` y) = ~` x `|` y.

Lemma leBC x y : x `\` y ~` y.

Lemma leCx x y : (~` x y) = (~` y x).

Lemma lexC x y : (x ~` y) = (y ~` x).

Lemma compl_joins (J : Type) (r : seq J) (P : {pred J}) (F : J L) :
   ~` (\join_(j <- r | P j) F j) = \meet_(j <- r | P j) ~` F j.

Lemma compl_meets (J : Type) (r : seq J) (P : {pred J}) (F : J L) :
   ~` (\meet_(j <- r | P j) F j) = \join_(j <- r | P j) ~` F j.

End CTBDistrLatticeTheory.
End CTBDistrLatticeTheory.







Implicit Types (x y z : T).

Let comparableT x y : x >=< y := le_total x y.

Fact meetUl : @left_distributive T T meet join.





Implicit Types (x y z : T).

Let comparableT x y : x >=< y := le_total x y.

Fact ltgtP x y :
  compare x y (min y x) (min x y) (max y x) (max x y)
              (y == x) (x == y) (x y) (x y) (x > y) (x < y).

Fact leP x y : le_xor_gt x y
  (min y x) (min x y) (max y x) (max x y) (x y) (y < x).

Definition meet := @min _ T.
Definition join := @max _ T.

Fact meetC : commutative meet.

Fact joinC : commutative join.

Fact meetA : associative meet.

Fact joinA : associative join.

Fact joinKI y x : meet x (join x y) = x.

Fact meetKU y x : join x (meet x y) = x.

Fact leEmeet x y : (x y) = (meet x y == x).




Fact le_refl : reflexive le.

Fact le_anti : antisymmetric le.

Fact le_trans : transitive le.






Fact meet_lel x y : meet x y meet y x.
Fact meetC : commutative meet.
Fact meet_leL {x y} : (meet x y) x.
Fact meet_leR {x y} : (meet x y) y.

Fact join_lel x y : join x y join y x.
Fact joinC : commutative join.
Fact join_leL {x y} : x (join x y).
Fact join_leR {x y} : y (join x y).

Fact meetA : associative meet.
Fact joinA : associative join.
Fact joinKI y x : meet x (join x y) = x.
Fact meetKU y x : join x (meet x y) = x.
Fact leEmeet x y : (x y) = (meet x y == x).





Fact le_refl : reflexive le.


Section GeneratedOrder.

Implicit Types (x y z : T').

Fact meetE x y : meet x y = x `&` y.
Fact joinE x y : join x y = x `|` y.
Fact meetC : commutative meet.
Fact joinC : commutative join.
Fact meetA : associative meet.
Fact joinA : associative join.
Fact joinKI y x : meet x (join x y) = x.
Fact meetKU y x : join x (meet x y) = x.
Fact meetUl : left_distributive meet join.
Fact meetxx : idempotent meet.
Fact le_def x y : x y = (meet x y == x).

End GeneratedOrder.





Fact lt_def x y : lt x y = (y != x) && le x y.

Fact meet_def_le x y : meet x y = if lt x y then x else y.

Fact join_def_le x y : join x y = if lt x y then y else x.

Fact le_anti : antisymmetric le.

Fact le_trans : transitive le.

Fact le_total : total le.


Lemma totalT : total (<=%O : rel T).

Module CancelPartial.
Section CancelPartial.
Variables (disp : unit) (T : choiceType).
Variables (disp' : unit) (T' : porderType disp') (f : T T').

Section PCan.
Variables (f' : T' option T) (f_can : pcancel f f').

Definition le (x y : T) := f x f y.
Definition lt (x y : T) := f x < f y.

Fact refl : reflexive le.
Fact anti : antisymmetric le.
Fact trans : transitive le.
Fact lt_def x y : lt x y = (y != x) && le x y.

Definition Pcan := isPOrder.Build disp T lt_def refl anti trans.

End PCan.

Definition Can f' (f_can : cancel f f') := Pcan (can_pcan f_can).

End CancelPartial.
End CancelPartial.

Notation PCanIsPartial := CancelPartial.Pcan.
Notation CanIsPartial := CancelPartial.Can.

#[deprecated(since="mathcomp 2.0.0", note="Use PCanIsPartial.")]
Notation PcanPartial := CancelPartial.Pcan.
#[deprecated(since="mathcomp 2.0.0", note="Use CanIsPartial.")]
Notation CanPartial := CancelPartial.Can.

#[export]
HB.instance Definition _ (disp : unit) (T : choiceType)
  (disp' : unit) (T' : porderType disp') (f : T T')
  (f' : T' option T) (f_can : pcancel f f') : isPOrder disp (pcan_type f_can) :=
  CancelPartial.Pcan disp (f_can : @pcancel _ (pcan_type f_can) f f').

#[export]
HB.instance Definition _ (disp : unit) (T : choiceType)
  (disp' : unit) (T' : porderType disp') (f : T T') (f' : T' T)
  (f_can : cancel f f') : isPOrder disp (can_type f_can) :=
  CancelPartial.Can disp (f_can : @cancel _ (can_type f_can) f f').

Section CancelTotal.
Variables (disp : unit) (T : choiceType).
Variables (disp' : unit) (T' : orderType disp') (f : T T').

Section PCan.

Variables (f' : T' option T) (f_can : pcancel f f').

#[local]
HB.instance Definition _ :=
   MonoTotal.Build disp (pcan_type f_can) (fun _ _erefl).

Definition PCanIsTotal : DistrLattice_isTotal _ (pcan_type f_can) :=
  Total.on (pcan_type f_can).

End PCan.

Section Can.

Variables (f' : T' T) (f_can : cancel f f').

#[local]
HB.instance Definition _ :=
   MonoTotal.Build disp (can_type f_can) (fun _ _erefl).

Definition CanIsTotal : DistrLattice_isTotal _ (can_type f_can) :=
  Total.on (can_type f_can).

End Can.
End CancelTotal.

#[deprecated(since="mathcomp 2.0.0", note="Use PCanIsTotal.")]
Notation PcanTotal := PCanIsTotal.
#[deprecated(since="mathcomp 2.0.0", note="Use CanIsTotal.")]
Notation CanTotal := CanIsTotal.



Definition meet (x y : T) := f' (meet (f x) (f y)).
Definition join (x y : T) := f' (join (f x) (f y)).

Lemma meetC : commutative meet.
Lemma joinC : commutative join.
Lemma meetA : associative meet.
Lemma joinA : associative join.
Lemma joinKI y x : meet x (join x y) = x.
Lemma meetKI y x : join x (meet x y) = x.
Lemma meet_eql x y : (x y) = (meet x y == x).






Lemma meetUl : left_distributive (meet : T T T) join.



Module CanExports.
#[deprecated(since="mathcomp 2.0.0", note="use Order.MonoTotal instead.")]
Notation MonoTotalMixin d T := (MonoTotal d T).
#[deprecated(since="mathcomp 2.0.0", note="use Order.PCanIsPartial instead.")]
Notation PcanPOrderMixin := CancelPartial.Pcan.
#[deprecated(since="mathcomp 2.0.0", note="use Order.CanIsPartial instead.")]
Notation CanPOrderMixin := CancelPartial.Can.
#[deprecated(since="mathcomp 2.0.0", note="use Order.PCanIsTotal instead.")]
Notation PcanOrderMixin := PCanIsTotal.
#[deprecated(since="mathcomp 2.0.0", note="use Order.CanIsTotal instead.")]
Notation CanOrderMixin := CanIsTotal.
#[deprecated(since="mathcomp 2.0.0", note="use Order.IsoLattice instead.")]
Notation IsoLatticeMixin d T := (IsoLattice d T).
#[deprecated(since="mathcomp 2.0.0", note="use Order.IsoDistrLattice instead.")]
Notation IsoDistrLatticeMixin d T := (IsoDistrLattice d T).
End CanExports.
Export CanExports.

Morphism hierarchy.

Definition order_morphism d (T : porderType d) d' (T' : porderType d')
  (f : T T') : Prop := {mono f : x y / x y}.



Module OrderMorphismExports.
Notation "{ 'omorphism' T -> T' }" :=
  (@OrderMorphism.type _ T%type _ T'%type) : type_scope.
End OrderMorphismExports.

Module Import OrderMorphismTheory.
Section OrderMorphismTheory.

Section Properties.

Variables (d : unit) (T : porderType d) (d' : unit) (T' : porderType d').
Variables (f : {omorphism T T'}).

Lemma omorph_le : {mono f : x y / x y}.

Lemma omorph_inj : injective f.

Lemma omorph_lt : {mono f : x y / x < y}.

End Properties.

Section IdCompFun.

Variables (d : unit) (T : porderType d) (d' : unit) (T' : porderType d').
Variables (d'' : unit) (T'' : porderType d'').
Variables (f : {omorphism T' T''}) (g : {omorphism T T'}).

Fact idfun_is_order_morphism : order_morphism (@idfun T).
#[export]
HB.instance Definition _ := isOrderMorphism.Build d T d T idfun
  idfun_is_order_morphism.

Fact comp_is_order_morphism : order_morphism (f \o g).
#[export]
HB.instance Definition _ := isOrderMorphism.Build d T d'' T'' (f \o g)
  comp_is_order_morphism.

End IdCompFun.

End OrderMorphismTheory.
End OrderMorphismTheory.

Definition meet_morphism d (T : latticeType d) d' (T' : latticeType d')
  (f : T T') : Prop := {morph f : x y / x `&` y}.

Definition join_morphism d (T : latticeType d) d' (T' : latticeType d')
  (f : T T') : Prop := {morph f : x y / x `|` y}.








Module LatticeMorphismExports.
Notation "{ 'mlmorphism' T -> T' }" :=
  (@MeetLatticeMorphism.type _ T%type _ T'%type) : type_scope.
Notation "{ 'jlmorphism' T -> T' }" :=
  (@JoinLatticeMorphism.type _ T%type _ T'%type) : type_scope.
Notation "{ 'lmorphism' T -> T' }" :=
  (@LatticeMorphism.type _ T%type _ T'%type) : type_scope.
Notation "[ 'mlmorphism' 'of' f 'as' g ]" :=
  (MeetLatticeMorphism.clone _ _ _ _ f%function g)
  (at level 0, format "[ 'mlmorphism' 'of' f 'as' g ]") : form_scope.
Notation "[ 'mlmorphism' 'of' f ]" :=
  (MeetLatticeMorphism.clone _ _ _ _ f%function _)
  (at level 0, format "[ 'mlmorphism' 'of' f ]") : form_scope.
Notation "[ 'jlmorphism' 'of' f 'as' g ]" :=
  (JoinLatticeMorphism.clone _ _ _ _ f%function g)
  (at level 0, format "[ 'jlmorphism' 'of' f 'as' g ]") : form_scope.
Notation "[ 'jlmorphism' 'of' f ]" :=
  (JoinLatticeMorphism.clone _ _ _ _ f%function _)
  (at level 0, format "[ 'jlmorphism' 'of' f ]") : form_scope.
Notation "[ 'lmorphism' 'of' f 'as' g ]" :=
  (LatticeMorphism.clone _ _ _ _ f%function g)
  (at level 0, format "[ 'lmorphism' 'of' f 'as' g ]") : form_scope.
Notation "[ 'lmorphism' 'of' f ]" :=
  (LatticeMorphism.clone _ _ _ _ f%function _)
  (at level 0, format "[ 'lmorphism' 'of' f ]") : form_scope.
End LatticeMorphismExports.

Module Import LatticeMorphismTheory.
Section LatticeMorphismTheory.

Section Properties.

Variables (d : unit) (T : latticeType d) (d' : unit) (T' : latticeType d').

Lemma omorphI (f : {mlmorphism T T'}) : {morph f : x y / x `&` y}.

Lemma omorphU (f : {jlmorphism T T'}) : {morph f : x y / x `|` y}.

End Properties.

Section IdCompFun.

Variables (d : unit) (T : latticeType d) (d' : unit) (T' : latticeType d').
Variables (d'' : unit) (T'' : latticeType d'').

Section MeetCompFun.

Variables (f : {mlmorphism T' T''}) (g : {mlmorphism T T'}).

Fact idfun_is_meet_morphism : meet_morphism (@idfun T).
#[export]
HB.instance Definition _ := isMeetLatticeMorphism.Build d T d T idfun
  idfun_is_meet_morphism.

Fact comp_is_meet_morphism : meet_morphism (f \o g).
#[export]
HB.instance Definition _ := isMeetLatticeMorphism.Build d T d'' T'' (f \o g)
  comp_is_meet_morphism.

End MeetCompFun.

Section JoinCompFun.

Variables (f : {jlmorphism T' T''}) (g : {jlmorphism T T'}).

Fact idfun_is_join_morphism : join_morphism (@idfun T).
#[export]
HB.instance Definition _ := isJoinLatticeMorphism.Build d T d T idfun
  idfun_is_join_morphism.

Fact comp_is_join_morphism : join_morphism (f \o g).
#[export]
HB.instance Definition _ := isJoinLatticeMorphism.Build d T d'' T'' (f \o g)
  comp_is_join_morphism.

End JoinCompFun.

End IdCompFun.

End LatticeMorphismTheory.
End LatticeMorphismTheory.






Module TBLatticeMorphismExports.
Notation "{ 'blmorphism' T -> T' }" :=
  (@BLatticeMorphism.type _ T%type _ T'%type) : type_scope.
Notation "{ 'tlmorphism' T -> T' }" :=
  (@TLatticeMorphism.type _ T%type _ T'%type) : type_scope.
Notation "{ 'tblmorphism' T -> T' }" :=
  (@TBLatticeMorphism.type _ T%type _ T'%type) : type_scope.
End TBLatticeMorphismExports.

Module Import BLatticeMorphismTheory.
Section BLatticeMorphismTheory.

Section Properties.

Variables (d : unit) (T : bLatticeType d) (d' : unit) (T' : bLatticeType d').
Variables (f : {blmorphism T T'}).

Lemma omorph0 : f \bot = \bot.

End Properties.

Section IdCompFun.

Variables (d : unit) (T : bLatticeType d) (d' : unit) (T' : bLatticeType d').
Variables (d'' : unit) (T'' : bLatticeType d'').
Variables (f : {blmorphism T' T''}) (g : {blmorphism T T'}).

Fact idfun_is_bottom_morphism : (@idfun T) \bot = \bot.
#[export]
HB.instance Definition _ := isBLatticeMorphism.Build d T d T idfun
  idfun_is_bottom_morphism.

Fact comp_is_bottom_morphism : (f \o g) \bot = \bot.
#[export]
HB.instance Definition _ := isBLatticeMorphism.Build d T d'' T'' (f \o g)
  comp_is_bottom_morphism.

End IdCompFun.

End BLatticeMorphismTheory.
End BLatticeMorphismTheory.

Module Import TLatticeMorphismTheory.
Section TLatticeMorphismTheory.

Section Properties.

Variables (d : unit) (T : tLatticeType d) (d' : unit) (T' : tLatticeType d').
Variables (f : {tlmorphism T T'}).

Lemma omorph1 : f \top = \top.

End Properties.

Section IdCompFun.

Variables (d : unit) (T : tLatticeType d) (d' : unit) (T' : tLatticeType d').
Variables (d'' : unit) (T'' : tLatticeType d'').
Variables (f : {tlmorphism T' T''}) (g : {tlmorphism T T'}).

Fact idfun_is_top_morphism : (@idfun T) \top = \top.
#[export]
HB.instance Definition _ := isTLatticeMorphism.Build d T d T idfun
  idfun_is_top_morphism.

Fact comp_is_top_morphism : (f \o g) \top = \top.
#[export]
HB.instance Definition _ := isTLatticeMorphism.Build d T d'' T'' (f \o g)
  comp_is_top_morphism.

End IdCompFun.

End TLatticeMorphismTheory.
End TLatticeMorphismTheory.

Module Import ClosedPredicates.
Section ClosedPredicates.

Variable (d : unit) (T : latticeType d).
Variable S : {pred T}.

Definition meet_closed := {in S &, u v, u `&` v \in S}.

Definition join_closed := {in S &, u v, u `|` v \in S}.

End ClosedPredicates.
End ClosedPredicates.

Mixins for stability properties





Structures for stability properties

#[short(type="meetLatticeClosed")]
HB.structure Definition MeetLatticeClosed d T :=
  {S of isMeetLatticeClosed d T S}.

#[short(type="joinLatticeClosed")]
HB.structure Definition JoinLatticeClosed d T :=
  {S of isJoinLatticeClosed d T S}.

#[short(type="latticeClosed")]
HB.structure Definition LatticeClosed d T :=
  {S of @MeetLatticeClosed d T S & @JoinLatticeClosed d T S}.

#[short(type="bLatticeClosed")]
HB.structure Definition BLatticeClosed d T := {S of isBLatticeClosed d T S}.

#[short(type="bJoinLatticeClosed")]
HB.structure Definition BJoinLatticeClosed d T :=
  {S of isBLatticeClosed d T S & @JoinLatticeClosed d T S}.

#[short(type="tLatticeClosed")]
HB.structure Definition TLatticeClosed d T := {S of isTLatticeClosed d T S}.

#[short(type="tMeetLatticeClosed")]
HB.structure Definition TMeetLatticeClosed d T :=
  {S of isTLatticeClosed d T S & @MeetLatticeClosed d T S}.

#[short(type="tbLatticeClosed")]
HB.structure Definition TBLatticeClosed d (T : tbLatticeType d) :=
  {S of @BLatticeClosed d T S & @TLatticeClosed d T S}.





Module Import LatticePred.
Section LatticePred.

Variables (d : unit) (T : latticeType d).

Lemma opredI (S : meetLatticeClosed T) : {in S &, u v, u `&` v \in S}.

Lemma opredU (S : joinLatticeClosed T) : {in S &, u v, u `|` v \in S}.

End LatticePred.

Section BLatticePred.

Variables (d : unit) (T : bLatticeType d).

Lemma opred0 (S : bLatticeClosed T) : \bot \in S.

Lemma opred_joins (S : bJoinLatticeClosed T) I r (P : pred I) F :
  ( i, P i F i \in S) \join_(i <- r | P i) F i \in S.

End BLatticePred.

Section TLatticePred.

Variables (d : unit) (T : tLatticeType d).

Lemma opred1 (S : tLatticeClosed T) : \top \in S.

Lemma opred_meets (S : tMeetLatticeClosed T) I r (P : pred I) F :
  ( i, P i F i \in S) \meet_(i <- r | P i) F i \in S.

End TLatticePred.
End LatticePred.


#[short(type="subPOrder")]
HB.structure Definition SubPOrder d (T : porderType d) S d' :=
  { U of SubChoice T S U & POrder d' U & isSubPOrder d T S d' U }.

Module Import SubPOrderTheory.
Section SubPOrderTheory.
Context (d : unit) (T : porderType d) (S : pred T).
Context (d' : unit) (U : SubPOrder.type S d').
Lemma leEsub x y : (x y) = (val x val y).
Lemma ltEsub x y : (x < y) = (val x < val y).
End SubPOrderTheory.
End SubPOrderTheory.


Fact valD : order_morphism (val : U T).

#[export]
HB.instance Definition _ d (T : porderType d) (S : pred T) (d' : unit)
  (U : subType S) := SubChoice_isSubPOrder.Build d T S d' (sub_type U).



#[short(type="subPOrderLattice")]
HB.structure Definition SubPOrderLattice d (T : latticeType d) S d' :=
  { U of @SubPOrder d T S d' U & Lattice d' U }.

#[short(type="subPOrderBLattice")]
HB.structure Definition SubPOrderBLattice d (T : latticeType d) S d' :=
  { U of @SubPOrderLattice d T S d' U & BLattice d' U }.

#[short(type="subPOrderTLattice")]
HB.structure Definition SubPOrderTLattice d (T : latticeType d) S d' :=
  { U of @SubPOrderLattice d T S d' U & TLattice d' U }.

#[short(type="subPOrderTBLattice")]
HB.structure Definition SubPOrderTBLattice d (T : latticeType d) S d' :=
  { U of @SubPOrderLattice d T S d' U & TBLattice d' U }.

#[short(type="meetSubLattice")]
HB.structure Definition MeetSubLattice d (T : latticeType d) S d' :=
  { U of @SubPOrderLattice d T S d' U & isMeetSubLattice d T S d' U }.

#[short(type="meetSubBLattice")]
HB.structure Definition MeetSubBLattice d (T : latticeType d) S d' :=
  { U of @MeetSubLattice d T S d' U & BLattice d' U }.

#[short(type="meetSubTLattice")]
HB.structure Definition MeetSubTLattice d (T : latticeType d) S d' :=
  { U of @MeetSubLattice d T S d' U & TLattice d' U }.

#[short(type="meetSubTBLattice")]
HB.structure Definition MeetSubTBLattice d (T : latticeType d) S d' :=
  { U of @MeetSubLattice d T S d' U & TBLattice d' U }.

#[short(type="joinSubLattice")]
HB.structure Definition JoinSubLattice d (T : latticeType d) S d' :=
  { U of @SubPOrderLattice d T S d' U & isJoinSubLattice d T S d' U }.

#[short(type="joinSubBLattice")]
HB.structure Definition JoinSubBLattice d (T : latticeType d) S d' :=
  { U of @JoinSubLattice d T S d' U & BLattice d' U }.

#[short(type="joinSubTLattice")]
HB.structure Definition JoinSubTLattice d (T : latticeType d) S d' :=
  { U of @JoinSubLattice d T S d' U & TLattice d' U }.

#[short(type="joinSubTBLattice")]
HB.structure Definition JoinSubTBLattice d (T : latticeType d) S d' :=
  { U of @JoinSubLattice d T S d' U & TBLattice d' U }.

#[short(type="subLattice")]
HB.structure Definition SubLattice d (T : latticeType d) S d' :=
  { U of @MeetSubLattice d T S d' U & @JoinSubLattice d T S d' U }.

#[short(type="subBLattice")]
HB.structure Definition SubBLattice d (T : latticeType d) S d' :=
  { U of @SubLattice d T S d' U & BLattice d' U }.

#[short(type="subTLattice")]
HB.structure Definition SubTLattice d (T : latticeType d) S d' :=
  { U of @SubLattice d T S d' U & TLattice d' U }.

#[short(type="subTBLattice")]
HB.structure Definition SubTBLattice d (T : latticeType d) S d' :=
  { U of @SubLattice d T S d' U & TBLattice d' U }.

#[export]
HB.instance Definition _ (d : unit) (T : latticeType d) (S : pred T)
    d' (U : MeetSubLattice.type S d') :=
  isMeetLatticeMorphism.Build d' U d T val valI_subproof.

#[export]
HB.instance Definition _ (d : unit) (T : latticeType d) (S : pred T)
    d' (U : JoinSubLattice.type S d') :=
  isJoinLatticeMorphism.Build d' U d T val valU_subproof.




Let inU v Sv : U := Sub v Sv.
Let meetU (u1 u2 : U) : U := inU (opredI (valP u1) (valP u2)).
Let joinU (u1 u2 : U) : U := inU (opredU (valP u1) (valP u2)).

Let meetUC : commutative meetU.
Let joinUC : commutative joinU.
Let meetUA : associative meetU.
Let joinUA : associative joinU.
Lemma joinUKI y x : meetU x (joinU x y) = x.
Let meetUKU y x : joinU x (meetU x y) = x.
Let le_meetU x y : (x y) = (meetU x y == x).

Fact valI : meet_morphism (val : U T).
Fact valU : join_morphism (val : U T).




#[short(type="bJoinSubLattice")]
HB.structure Definition BJoinSubLattice d (T : bLatticeType d) S d' :=
  { U of @JoinSubLattice d T S d' U & BLattice d' U & isBSubLattice d T S d' U }.

#[short(type="bJoinSubTLattice")]
HB.structure Definition BJoinSubTLattice d (T : bLatticeType d) S d' :=
  { U of @BJoinSubLattice d T S d' U & TBLattice d' U }.

#[short(type="bSubLattice")]
HB.structure Definition BSubLattice d (T : bLatticeType d) S d' :=
  { U of @SubLattice d T S d' U & @BJoinSubLattice d T S d' U }.

#[short(type="bSubTLattice")]
HB.structure Definition BSubTLattice d (T : bLatticeType d) S d' :=
  { U of @BSubLattice d T S d' U & TBLattice d' U }.

#[export]
HB.instance Definition _ (d : unit) (T : bLatticeType d) (S : pred T)
    d' (U : BJoinSubLattice.type S d') :=
  isBLatticeMorphism.Build d' U d T val val0_subproof.



Let inU v Sv : U := Sub v Sv.
Let zeroU : U := inU opred0_subproof.

Fact le0x x : zeroU x.

Fact val0 : (val : U T) \bot = \bot.




#[short(type="tMeetSubLattice")]
HB.structure Definition TMeetSubLattice d (T : tLatticeType d) S d' :=
  { U of @MeetSubLattice d T S d' U & TLattice d' U & isTSubLattice d T S d' U }.

#[short(type="tMeetSubBLattice")]
HB.structure Definition TMeetSubBLattice d (T : tLatticeType d) S d' :=
  { U of @TMeetSubLattice d T S d' U & TBLattice d' U }.

#[short(type="tSubLattice")]
HB.structure Definition TSubLattice d (T : tLatticeType d) S d' :=
  { U of @SubLattice d T S d' U & @TMeetSubLattice d T S d' U }.

#[short(type="tSubBLattice")]
HB.structure Definition TSubBLattice d (T : tLatticeType d) S d' :=
  { U of @TSubLattice d T S d' U & TBLattice d' U }.

#[export]
HB.instance Definition _ (d : unit) (T : tLatticeType d) (S : pred T)
    d' (U : TMeetSubLattice.type S d') :=
  isTLatticeMorphism.Build d' U d T val val1_subproof.



Let inU v Sv : U := Sub v Sv.
Let oneU : U := inU opred1_subproof.

Fact lex1 x : x oneU.

Fact val1 : (val : U T) \top = \top.



#[short(type="tbSubLattice")]
HB.structure Definition TBSubLattice d (T : tbLatticeType d) S d' :=
  { U of @BSubLattice d T S d' U & @TSubLattice d T S d' U}.

#[export]
HB.instance Definition _ (d : unit) (T : tbLatticeType d) (S : pred T) d'
    (U : TBSubLattice.type S d') := BLatticeMorphism.on (val : U T).





#[short(type="subOrder")]
HB.structure Definition SubOrder d (T : orderType d) S d' :=
  { U of @SubLattice d T S d' U & Total d' U }.


Lemma totalU : total (<=%O : rel U).


Fact opredI : meet_closed S.
Fact opredU : join_closed S.



Module SubOrderExports.

Notation "[ 'SubChoice_isSubPOrder' 'of' U 'by' <: ]" :=
  (SubChoice_isSubPOrder.Build _ _ _ _ U)
  (at level 0, format "[ 'SubChoice_isSubPOrder' 'of' U 'by' <: ]")
  : form_scope.
Notation "[ 'SubChoice_isSubPOrder' 'of' U 'by' <: 'with' disp ]" :=
  (SubChoice_isSubPOrder.Build _ _ _ disp U)
  (at level 0, format "[ 'SubChoice_isSubPOrder' 'of' U 'by' <: 'with' disp ]")
  : form_scope.
Notation "[ 'SubPOrder_isSubLattice' 'of' U 'by' <: ]" :=
  (SubPOrder_isSubLattice.Build _ _ _ _ U (@opredI _ _ _) (@opredU _ _ _))
  (at level 0, format "[ 'SubPOrder_isSubLattice' 'of' U 'by' <: ]")
  : form_scope.
Notation "[ 'SubPOrder_isSubLattice' 'of' U 'by' <: 'with' disp ]" :=
  (SubPOrder_isSubLattice.Build _ _ _ disp U (@opredI _ _ _) (@opredU _ _ _))
  (at level 0, format "[ 'SubPOrder_isSubLattice' 'of' U 'by' <: 'with' disp ]")
  : form_scope.
Notation "[ 'SubChoice_isSubLattice' 'of' U 'by' <: ]" :=
  (SubChoice_isSubLattice.Build _ _ _ _ U (@opredI _ _ _) (@opredU _ _ _))
  (at level 0, format "[ 'SubChoice_isSubLattice' 'of' U 'by' <: ]")
    : form_scope.
Notation "[ 'SubChoice_isSubLattice' 'of' U 'by' <: 'with' disp ]" :=
  (SubChoice_isSubLattice.Build _ _ _ disp U (@opredI _ _ _) (@opredU _ _ _))
  (at level 0, format "[ 'SubChoice_isSubLattice' 'of' U 'by' <: 'with' disp ]")
    : form_scope.
Notation "[ 'SubPOrder_isBSubLattice' 'of' U 'by' <: ]" :=
  (SubPOrder_isBSubLattice.Build _ _ _ _ U (opred0 _))
  (at level 0, format "[ 'SubPOrder_isBSubLattice' 'of' U 'by' <: ]")
  : form_scope.
Notation "[ 'SubPOrder_isBSubLattice' 'of' U 'by' <: 'with' disp ]" :=
  (SubPOrder_isBSubLattice.Build _ _ _ disp U (opred0 _))
  (at level 0, format "[ 'SubPOrder_isBSubLattice' 'of' U 'by' <: 'with' disp ]")
  : form_scope.
Notation "[ 'SubChoice_isBSubLattice' 'of' U 'by' <: ]" :=
  (SubChoice_isBSubLattice.Build _ _ _ _ U
     (@opredI _ _ _) (@opredU _ _ _) (opred0 _))
  (at level 0, format "[ 'SubChoice_isBSubLattice' 'of' U 'by' <: ]")
  : form_scope.
Notation "[ 'SubChoice_isBSubLattice' 'of' U 'by' <: 'with' disp ]" :=
  (SubChoice_isBSubLattice.Build _ _ _ disp U
     (@opredI _ _ _) (@opredU _ _ _) (opred0 _))
  (at level 0, format "[ 'SubChoice_isBSubLattice' 'of' U 'by' <: 'with' disp ]")
  : form_scope.
Notation "[ 'SubPOrder_isTSubLattice' 'of' U 'by' <: ]" :=
  (SubPOrder_isTSubLattice.Build _ _ _ _ U (opred1 _))
  (at level 0, format "[ 'SubPOrder_isTSubLattice' 'of' U 'by' <: ]")
  : form_scope.
Notation "[ 'SubPOrder_isTSubLattice' 'of' U 'by' <: 'with' disp ]" :=
  (SubPOrder_isTSubLattice.Build _ _ _ disp U (opred1 _))
  (at level 0, format "[ 'SubPOrder_isTSubLattice' 'of' U 'by' <: 'with' disp ]")
  : form_scope.
Notation "[ 'SubChoice_isTSubLattice' 'of' U 'by' <: ]" :=
  (SubChoice_isTSubLattice.Build _ _ _ _ U
     (@opredI _ _ _) (@opredU _ _ _) (opred1 _))
  (at level 0, format "[ 'SubChoice_isTSubLattice' 'of' U 'by' <: ]")
  : form_scope.
Notation "[ 'SubChoice_isTSubLattice' 'of' U 'by' <: 'with' disp ]" :=
  (SubChoice_isTSubLattice.Build _ _ _ disp U
     (@opredI _ _ _) (@opredU _ _ _) (opred1 _))
  (at level 0, format "[ 'SubChoice_isTSubLattice' 'of' U 'by' <: 'with' disp ]")
  : form_scope.
Notation "[ 'SubPOrder_isTBSubLattice' 'of' U 'by' <: ]" :=
  (SubPOrder_isTBSubLattice.Build _ _ _ _ U (opred0 _) (opred1 _))
  (at level 0, format "[ 'SubPOrder_isTBSubLattice' 'of' U 'by' <: ]")
  : form_scope.
Notation "[ 'SubPOrder_isTBSubLattice' 'of' U 'by' <: 'with' disp ]" :=
  (SubPOrder_isTBSubLattice.Build _ _ _ disp U (opred0 _) (opred1 _))
  (at level 0, format "[ 'SubPOrder_isTBSubLattice' 'of' U 'by' <: 'with' disp ]")
  : form_scope.
Notation "[ 'SubChoice_isTBSubLattice' 'of' U 'by' <: ]" :=
  (SubChoice_isTBSubLattice.Build _ _ _ _ U
     (@opredI _ _ _) (@opredU _ _ _) (opred0 _) (opred1 _))
  (at level 0, format "[ 'SubChoice_isTBSubLattice' 'of' U 'by' <: ]")
  : form_scope.
Notation "[ 'SubChoice_isTBSubLattice' 'of' U 'by' <: 'with' disp ]" :=
  (SubChoice_isTBSubLattice.Build _ _ _ disp U
     (@opredI _ _ _) (@opredU _ _ _) (opred0 _) (opred1 _))
  (at level 0, format "[ 'SubChoice_isTBSubLattice' 'of' U 'by' <: 'with' disp ]")
  : form_scope.
Notation "[ 'SubLattice_isSubOrder' 'of' U 'by' <: ]" :=
  (SubLattice_isSubOrder.Build _ _ _ _ U)
  (at level 0, format "[ 'SubLattice_isSubOrder' 'of' U 'by' <: ]")
  : form_scope.
Notation "[ 'SubLattice_isSubOrder' 'of' U 'by' <: 'with' disp ]" :=
  (SubLattice_isSubOrder.Build _ _ _ disp U)
  (at level 0, format "[ 'SubLattice_isSubOrder' 'of' U 'by' <: 'with' disp ]")
  : form_scope.
Notation "[ 'SubPOrder_isSubOrder' 'of' U 'by' <: ]" :=
  (SubPOrder_isSubOrder.Build _ _ _ _ U)
  (at level 0, format "[ 'SubPOrder_isSubOrder' 'of' U 'by' <: ]")
  : form_scope.
Notation "[ 'SubPOrder_isSubOrder' 'of' U 'by' <: 'with' disp ]" :=
  (SubPOrder_isSubOrder.Build _ _ _ disp U)
  (at level 0, format "[ 'SubPOrder_isSubOrder' 'of' U 'by' <: 'with' disp ]")
  : form_scope.
Notation "[ 'SubChoice_isSubOrder' 'of' U 'by' <: ]" :=
  (SubChoice_isSubOrder.Build _ _ _ _ U)
  (at level 0, format "[ 'SubChoice_isSubOrder' 'of' U 'by' <: ]")
  : form_scope.
Notation "[ 'SubChoice_isSubOrder' 'of' U 'by' <: 'with' disp ]" :=
  (SubChoice_isSubOrder.Build _ _ _ disp U)
  (at level 0, format "[ 'SubChoice_isSubOrder' 'of' U 'by' <: 'with' disp ]")
  : form_scope.

End SubOrderExports.

Module DeprecatedSubOrder.

Section Total.
Context {disp : unit} {T : orderType disp} (P : {pred T}) (sT : subType P).

#[export]
HB.instance Definition _ :=
  SubPOrder_isSubOrder.Build disp T P disp (sub_type sT).

End Total.

Module Exports.
Notation "[ 'POrder' 'of' T 'by' <: ]" :=
  (POrder.copy T%type (sub_type T%type))
  (at level 0, format "[ 'POrder' 'of' T 'by' <: ]") : form_scope.
Notation "[ 'Order' 'of' T 'by' <: ]" :=
  (Total.copy T%type (sub_type T%type))
  (at level 0, only parsing) : form_scope.
End Exports.
End DeprecatedSubOrder.

INSTANCES Instances on nat This is an example of creation of multiple instances on the same type, with distinct displays, on the example of natural numbers. We declare two distinct canonical orders:
  • leq which is total, and where meet and join are minn and maxn, on nat
  • dvdn which is partial, and where meet and join are gcdn and lcmn, on a "copy" of nat we name natdiv
The Module NatOrder defines leq as the canonical order on the type nat, i.e., without creating a "copy". We define and use nat_display and proceed like standard canonical structure declaration, except we use this display. We also use a single factory LeOrderMixin to instantiate three different canonical declarations porderType, distrLatticeType, orderType We finish by providing theorems to convert the operations of ordered and lattice types to their definition without structure abstraction.

Module NatOrder.
Section NatOrder.

Fact nat_display : unit.

Lemma ltn_def x y : (x < y)%N = (y != x) && (x y)%N.

#[export]
HB.instance Definition _ :=
  isOrder.Build nat_display nat ltn_def (fun _ _erefl) (fun _ _erefl)
                anti_leq leq_trans leq_total.

#[export]
HB.instance Definition _ := hasBottom.Build nat_display nat leq0n.

Lemma leEnat : le = leq.
Lemma ltEnat : lt = ltn.
Lemma minEnat : min = minn.
Lemma maxEnat : max = maxn.
Lemma botEnat : \bot = 0%N :> nat.

End NatOrder.

Module Exports.
Definition leEnat := leEnat.
Definition ltEnat := ltEnat.
Definition minEnat := minEnat.
Definition maxEnat := maxEnat.
Definition botEnat := botEnat.
End Exports.
End NatOrder.

Module NatMonotonyTheory.
Section NatMonotonyTheory.

Context {disp : unit} {T : porderType disp}.
Variables (D : {pred nat}) (f : nat T).
Hypothesis Dconvex : {in D &, i j k, i < k < j k \in D}.

Lemma homo_ltn_lt_in : {in D, i, i.+1 \in D f i < f i.+1}
  {in D &, {homo f : i j / i < j}}.

Lemma incn_inP : {in D, i, i.+1 \in D f i < f i.+1}
  {in D &, {mono f : i j / i j}}.

Lemma nondecn_inP : {in D, i, i.+1 \in D f i f i.+1}
  {in D &, {homo f : i j / i j}}.

Lemma nhomo_ltn_lt_in : {in D, i, i.+1 \in D f i > f i.+1}
  {in D &, {homo f : i j /~ i < j}}.

Lemma decn_inP : {in D, i, i.+1 \in D f i > f i.+1}
  {in D &, {mono f : i j /~ i j}}.

Lemma nonincn_inP : {in D, i, i.+1 \in D f i f i.+1}
  {in D &, {homo f : i j /~ i j}}.

Lemma homo_ltn_lt : ( i, f i < f i.+1) {homo f : i j / i < j}.

Lemma incnP : ( i, f i < f i.+1) {mono f : i j / i j}.

Lemma nondecnP : ( i, f i f i.+1) {homo f : i j / i j}.

Lemma nhomo_ltn_lt : ( i, f i > f i.+1) {homo f : i j /~ i < j}.

Lemma decnP : ( i, f i > f i.+1) {mono f : i j /~ i j}.

Lemma nonincnP : ( i, f i f i.+1) {homo f : i j /~ i j}.

End NatMonotonyTheory.
Arguments homo_ltn_lt_in {disp T} [D f].
Arguments incn_inP {disp T} [D f].
Arguments nondecn_inP {disp T} [D f].
Arguments nhomo_ltn_lt_in {disp T} [D f].
Arguments decn_inP {disp T} [D f].
Arguments nonincn_inP {disp T} [D f].
Arguments homo_ltn_lt {disp T} [f].
Arguments incnP {disp T} [f].
Arguments nondecnP {disp T} [f].
Arguments nhomo_ltn_lt {disp T} [f].
Arguments decnP {disp T} [f].
Arguments nonincnP {disp T} [f].

End NatMonotonyTheory.

The Module DvdSyntax introduces a new set of notations using the newly created display dvd_display. We first define the display as an opaque definition of type unit, and we use it as the first argument of the operator which display we want to change from the default one (here le, lt, dvd sdvd, meet, join, top and bottom, as well as big op notations on gcd and lcm). This notations will now be used for any ordered type which first parameter is set to dvd_display.

Fact dvd_display : unit.

Module DvdSyntax.

Notation dvd := (@le dvd_display _).
Notation "@ 'dvd' T" :=
  (@le dvd_display T) (at level 10, T at level 8, only parsing) : function_scope.
Notation sdvd := (@lt dvd_display _).
Notation "@ 'sdvd' T" :=
  (@lt dvd_display T) (at level 10, T at level 8, only parsing) : function_scope.

Notation "x %| y" := (dvd x y) : order_scope.
Notation "x %<| y" := (sdvd x y) : order_scope.

Notation gcd := (@meet dvd_display _).
Notation "@ 'gcd' T" :=
  (@meet dvd_display T) (at level 10, T at level 8, only parsing) : function_scope.
Notation lcm := (@join dvd_display _).
Notation "@ 'lcm' T" :=
  (@join dvd_display T) (at level 10, T at level 8, only parsing) : function_scope.

Notation nat0 := (@top dvd_display _).
Notation nat1 := (@bottom dvd_display _).

Notation "\gcd_ ( i <- r | P ) F" :=
  (\big[gcd/nat0]_(i <- r | P%B) F%O) : order_scope.
Notation "\gcd_ ( i <- r ) F" :=
  (\big[gcd/nat0]_(i <- r) F%O) : order_scope.
Notation "\gcd_ ( i | P ) F" :=
  (\big[gcd/nat0]_(i | P%B) F%O) : order_scope.
Notation "\gcd_ i F" :=
  (\big[gcd/nat0]_i F%O) : order_scope.
Notation "\gcd_ ( i : I | P ) F" :=
  (\big[gcd/nat0]_(i : I | P%B) F%O) (only parsing) :
  order_scope.
Notation "\gcd_ ( i : I ) F" :=
  (\big[gcd/nat0]_(i : I) F%O) (only parsing) : order_scope.
Notation "\gcd_ ( m <= i < n | P ) F" :=
  (\big[gcd/nat0]_(m i < n | P%B) F%O) : order_scope.
Notation "\gcd_ ( m <= i < n ) F" :=
  (\big[gcd/nat0]_(m i < n) F%O) : order_scope.
Notation "\gcd_ ( i < n | P ) F" :=
  (\big[gcd/nat0]_(i < n | P%B) F%O) : order_scope.
Notation "\gcd_ ( i < n ) F" :=
  (\big[gcd/nat0]_(i < n) F%O) : order_scope.
Notation "\gcd_ ( i 'in' A | P ) F" :=
  (\big[gcd/nat0]_(i in A | P%B) F%O) : order_scope.
Notation "\gcd_ ( i 'in' A ) F" :=
  (\big[gcd/nat0]_(i in A) F%O) : order_scope.

Notation "\lcm_ ( i <- r | P ) F" :=
  (\big[lcm/nat1]_(i <- r | P%B) F%O) : order_scope.
Notation "\lcm_ ( i <- r ) F" :=
  (\big[lcm/nat1]_(i <- r) F%O) : order_scope.
Notation "\lcm_ ( i | P ) F" :=
  (\big[lcm/nat1]_(i | P%B) F%O) : order_scope.
Notation "\lcm_ i F" :=
  (\big[lcm/nat1]_i F%O) : order_scope.
Notation "\lcm_ ( i : I | P ) F" :=
  (\big[lcm/nat1]_(i : I | P%B) F%O) (only parsing) :
  order_scope.
Notation "\lcm_ ( i : I ) F" :=
  (\big[lcm/nat1]_(i : I) F%O) (only parsing) : order_scope.
Notation "\lcm_ ( m <= i < n | P ) F" :=
  (\big[lcm/nat1]_(m i < n | P%B) F%O) : order_scope.
Notation "\lcm_ ( m <= i < n ) F" :=
  (\big[lcm/nat1]_(m i < n) F%O) : order_scope.
Notation "\lcm_ ( i < n | P ) F" :=
  (\big[lcm/nat1]_(i < n | P%B) F%O) : order_scope.
Notation "\lcm_ ( i < n ) F" :=
  (\big[lcm/nat1]_(i < n) F%O) : order_scope.
Notation "\lcm_ ( i 'in' A | P ) F" :=
  (\big[lcm/nat1]_(i in A | P%B) F%O) : order_scope.
Notation "\lcm_ ( i 'in' A ) F" :=
  (\big[lcm/nat1]_(i in A) F%O) : order_scope.

End DvdSyntax.

The Module NatDvd defines dvdn as the canonical order on NatDvd.t, which is abbreviated using the notation natdvd at the end of the module. We use the newly defined dvd_display, described above. This looks like standard canonical structure declaration, except we use a display and we declare it on a "copy" of the type. We first recover structures that are common to both nat and natdiv (eqType, choiceType, countType) through the clone mechanisms, then we use a single factory MeetJoinMixin to instantiate both porderType and distrLatticeType canonical structures, and end with top and bottom. We finish by providing theorems to convert the operations of ordered and lattice types to their definition without structure abstraction.

Module NatDvd.
Section NatDvd.

Implicit Types m n p : nat.

Lemma lcmnn n : lcmn n n = n.

Lemma le_def m n : m %| n = (gcdn m n == m)%N.

Lemma joinKI n m : gcdn m (lcmn m n) = m.

Lemma meetKU n m : lcmn m (gcdn m n) = m.

Lemma meetUl : left_distributive gcdn lcmn.

Definition t := nat.

#[export]
HB.instance Definition _ := Choice.copy t nat.

Note that this where the dvd_display is associated with the type NatDvd.t.
#[export]
HB.instance Definition _ := isMeetJoinDistrLattice.Build
  dvd_display t le_def (fun _ _erefl)
  gcdnC lcmnC gcdnA lcmnA joinKI meetKU meetUl gcdnn.
NatDvd.t is associated below with the notation "natdvd".

#[export]
HB.instance Definition _ := hasBottom.Build _ t (dvd1n : m : t, (1 %| m)).

#[export]
HB.instance Definition _ := hasTop.Build _ t (dvdn0 : m : t, (m %| 0)).

Import DvdSyntax.
Lemma dvdE : dvd = dvdn :> rel t.
Lemma sdvdE (m n : t) : m %<| n = (n != m) && (m %| n).
Lemma gcdE : gcd = gcdn :> (t t t).
Lemma lcmE : lcm = lcmn :> (t t t).
Lemma nat1E : nat1 = 1%N :> t.
Lemma nat0E : nat0 = 0%N :> t.

End NatDvd.
Module Exports.
Notation natdvd := t.
Definition dvdEnat := dvdE.
Definition sdvdEnat := sdvdE.
Definition gcdEnat := gcdE.
Definition lcmEnat := lcmE.
Definition nat1E := nat1E.
Definition nat0E := nat0E.
End Exports.
End NatDvd.

Instances on ordinal

Module OrdinalOrder.
Section OrdinalOrder.

Fact ord_display : unit.

Section PossiblyTrivial.
Variable (n : nat).

#[export]
HB.instance Definition _ :=
  [SubChoice_isSubOrder of 'I_n by <: with ord_display].

Lemma leEord : (le : rel 'I_n) = leq.
Lemma ltEord : (lt : rel 'I_n) = (fun m nm < n)%N.
End PossiblyTrivial.

Section NonTrivial.
Variable (n' : nat).
Let n := n'.+1.

#[export]
HB.instance Definition _ :=
   hasBottom.Build _ 'I_n (leq0n : x, ord0 x).
#[export]
HB.instance Definition _ :=
   hasTop.Build _ 'I_n (@leq_ord _ : x, x ord_max).

Lemma botEord : \bot = ord0.
Lemma topEord : \top = ord_max.

End NonTrivial.

End OrdinalOrder.

Module Exports.
Definition leEord := leEord.
Definition ltEord := ltEord.
Definition botEord := botEord.
Definition topEord := topEord.
End Exports.
End OrdinalOrder.

Instances on bool

Module BoolOrder.
Section BoolOrder.
Implicit Types (x y : bool).

Fact bool_display : unit.

Fact andbE x y : x && y = if (x < y)%N then x else y.

Fact orbE x y : x || y = if (x < y)%N then y else x.

Fact ltn_def x y : (x < y)%N = (y != x) && (x y)%N.

Fact anti : antisymmetric (leq : rel bool).

Definition sub x y := x && ~~ y.

Lemma subKI x y : y && sub x y = false.
Lemma joinIB x y : (x && y) || sub x y = x.

#[export] HB.instance Definition _ := @isOrder.Build bool_display bool
   _ _ andb orb ltn_def andbE orbE anti leq_trans leq_total.
#[export] HB.instance Definition _ := @hasBottom.Build _ bool false leq0n.
#[export] HB.instance Definition _ := @hasTop.Build _ bool true leq_b1.
#[export] HB.instance Definition _ := @hasRelativeComplement.Build _ bool sub subKI joinIB.
#[export] HB.instance Definition _ := @hasComplement.Build _ bool
  negb (fun xerefl : ~~ x = sub true x).

Lemma leEbool : le = (leq : rel bool).
Lemma ltEbool x y : (x < y) = (x < y)%N.
Lemma andEbool : meet = andb.
Lemma orEbool : meet = andb.
Lemma subEbool x y : x `\` y = x && ~~ y.
Lemma complEbool : compl = negb.

End BoolOrder.
Module Exports.
Definition leEbool := leEbool.
Definition ltEbool := ltEbool.
Definition andEbool := andEbool.
Definition orEbool := orEbool.
Definition subEbool := subEbool.
Definition complEbool := complEbool.
End Exports.
End BoolOrder.

Definition of prod_display

Fact prod_display : unit.

Module Import ProdSyntax.

Notation "<=^p%O" := (@le prod_display _) : function_scope.
Notation ">=^p%O" := (@ge prod_display _) : function_scope.
Notation ">=^p%O" := (@ge prod_display _) : function_scope.
Notation "<^p%O" := (@lt prod_display _) : function_scope.
Notation ">^p%O" := (@gt prod_display _) : function_scope.
Notation "<?=^p%O" := (@leif prod_display _) : function_scope.
Notation ">=<^p%O" := (@comparable prod_display _) : function_scope.
Notation "><^p%O" := (fun x y~~ (@comparable prod_display _ x y)) :
  function_scope.

Notation "<=^p y" := (>=^p%O y) : order_scope.
Notation "<=^p y :> T" := (<=^p (y : T)) (only parsing) : order_scope.
Notation ">=^p y" := (<=^p%O y) : order_scope.
Notation ">=^p y :> T" := (>=^p (y : T)) (only parsing) : order_scope.

Notation "<^p y" := (>^p%O y) : order_scope.
Notation "<^p y :> T" := (<^p (y : T)) (only parsing) : order_scope.
Notation ">^p y" := (<^p%O y) : order_scope.
Notation ">^p y :> T" := (>^p (y : T)) (only parsing) : order_scope.

Notation "x <=^p y" := (<=^p%O x y) : order_scope.
Notation "x <=^p y :> T" := ((x : T) <=^p (y : T)) (only parsing) : order_scope.
Notation "x >=^p y" := (y <=^p x) (only parsing) : order_scope.
Notation "x >=^p y :> T" := ((x : T) >=^p (y : T)) (only parsing) : order_scope.

Notation "x <^p y" := (<^p%O x y) : order_scope.
Notation "x <^p y :> T" := ((x : T) <^p (y : T)) (only parsing) : order_scope.
Notation "x >^p y" := (y <^p x) (only parsing) : order_scope.
Notation "x >^p y :> T" := ((x : T) >^p (y : T)) (only parsing) : order_scope.

Notation "x <=^p y <=^p z" := ((x <=^p y) && (y <=^p z)) : order_scope.
Notation "x <^p y <=^p z" := ((x <^p y) && (y <=^p z)) : order_scope.
Notation "x <=^p y <^p z" := ((x <=^p y) && (y <^p z)) : order_scope.
Notation "x <^p y <^p z" := ((x <^p y) && (y <^p z)) : order_scope.

Notation "x <=^p y ?= 'iff' C" := (<?=^p%O x y C) : order_scope.
Notation "x <=^p y ?= 'iff' C :> T" := ((x : T) <=^p (y : T) ?= iff C)
  (only parsing) : order_scope.

Notation ">=<^p y" := [pred x | >=<^p%O x y] : order_scope.
Notation ">=<^p y :> T" := (>=<^p (y : T)) (only parsing) : order_scope.
Notation "x >=<^p y" := (>=<^p%O x y) : order_scope.

Notation "><^p y" := [pred x | ~~ (>=<^p%O x y)] : order_scope.
Notation "><^p y :> T" := (><^p (y : T)) (only parsing) : order_scope.
Notation "x ><^p y" := (~~ (><^p%O x y)) : order_scope.

The following Local Notations are here to define the \join^p_ and \meet^p_ notations later. Do not remove them.

Notation "x `&^p` y" := (meet x y) : order_scope.
Notation "x `|^p` y" := (join x y) : order_scope.

Notation "\join^p_ ( i <- r | P ) F" :=
  (\big[join / \bot]_(i <- r | P%B) F%O) : order_scope.
Notation "\join^p_ ( i <- r ) F" :=
  (\big[join / \bot]_(i <- r) F%O) : order_scope.
Notation "\join^p_ ( i | P ) F" :=
  (\big[join / \bot]_(i | P%B) F%O) : order_scope.
Notation "\join^p_ i F" :=
  (\big[join / \bot]_i F%O) : order_scope.
Notation "\join^p_ ( i : I | P ) F" :=
  (\big[join / \bot]_(i : I | P%B) F%O) (only parsing) : order_scope.
Notation "\join^p_ ( i : I ) F" :=
  (\big[join / \bot]_(i : I) F%O) (only parsing) : order_scope.
Notation "\join^p_ ( m <= i < n | P ) F" :=
 (\big[join / \bot]_(m i < n | P%B) F%O) : order_scope.
Notation "\join^p_ ( m <= i < n ) F" :=
 (\big[join / \bot]_(m i < n) F%O) : order_scope.
Notation "\join^p_ ( i < n | P ) F" :=
 (\big[join / \bot]_(i < n | P%B) F%O) : order_scope.
Notation "\join^p_ ( i < n ) F" :=
 (\big[join / \bot]_(i < n) F%O) : order_scope.
Notation "\join^p_ ( i 'in' A | P ) F" :=
 (\big[join / \bot]_(i in A | P%B) F%O) : order_scope.
Notation "\join^p_ ( i 'in' A ) F" :=
 (\big[join / \bot]_(i in A) F%O) : order_scope.

Notation "\meet^p_ ( i <- r | P ) F" :=
  (\big[meet / \top]_(i <- r | P%B) F%O) : order_scope.
Notation "\meet^p_ ( i <- r ) F" :=
  (\big[meet / \top]_(i <- r) F%O) : order_scope.
Notation "\meet^p_ ( i | P ) F" :=
  (\big[meet / \top]_(i | P%B) F%O) : order_scope.
Notation "\meet^p_ i F" :=
  (\big[meet / \top]_i F%O) : order_scope.
Notation "\meet^p_ ( i : I | P ) F" :=
  (\big[meet / \top]_(i : I | P%B) F%O) (only parsing) : order_scope.
Notation "\meet^p_ ( i : I ) F" :=
  (\big[meet / \top]_(i : I) F%O) (only parsing) : order_scope.
Notation "\meet^p_ ( m <= i < n | P ) F" :=
 (\big[meet / \top]_(m i < n | P%B) F%O) : order_scope.
Notation "\meet^p_ ( m <= i < n ) F" :=
 (\big[meet / \top]_(m i < n) F%O) : order_scope.
Notation "\meet^p_ ( i < n | P ) F" :=
 (\big[meet / \top]_(i < n | P%B) F%O) : order_scope.
Notation "\meet^p_ ( i < n ) F" :=
 (\big[meet / \top]_(i < n) F%O) : order_scope.
Notation "\meet^p_ ( i 'in' A | P ) F" :=
 (\big[meet / \top]_(i in A | P%B) F%O) : order_scope.
Notation "\meet^p_ ( i 'in' A ) F" :=
 (\big[meet / \top]_(i in A) F%O) : order_scope.

End ProdSyntax.

Definition of lexi_display

Fact lexi_display : unit.

Module Import LexiSyntax.

Notation "<=^l%O" := (@le lexi_display _) : function_scope.
Notation ">=^l%O" := (@ge lexi_display _) : function_scope.
Notation ">=^l%O" := (@ge lexi_display _) : function_scope.
Notation "<^l%O" := (@lt lexi_display _) : function_scope.
Notation ">^l%O" := (@gt lexi_display _) : function_scope.
Notation "<?=^l%O" := (@leif lexi_display _) : function_scope.
Notation ">=<^l%O" := (@comparable lexi_display _) : function_scope.
Notation "><^l%O" := (fun x y~~ (@comparable lexi_display _ x y)) :
  function_scope.

Notation "<=^l y" := (>=^l%O y) : order_scope.
Notation "<=^l y :> T" := (<=^l (y : T)) (only parsing) : order_scope.
Notation ">=^l y" := (<=^l%O y) : order_scope.
Notation ">=^l y :> T" := (>=^l (y : T)) (only parsing) : order_scope.

Notation "<^l y" := (>^l%O y) : order_scope.
Notation "<^l y :> T" := (<^l (y : T)) (only parsing) : order_scope.
Notation ">^l y" := (<^l%O y) : order_scope.
Notation ">^l y :> T" := (>^l (y : T)) (only parsing) : order_scope.

Notation "x <=^l y" := (<=^l%O x y) : order_scope.
Notation "x <=^l y :> T" := ((x : T) <=^l (y : T)) (only parsing) : order_scope.
Notation "x >=^l y" := (y <=^l x) (only parsing) : order_scope.
Notation "x >=^l y :> T" := ((x : T) >=^l (y : T)) (only parsing) : order_scope.

Notation "x <^l y" := (<^l%O x y) : order_scope.
Notation "x <^l y :> T" := ((x : T) <^l (y : T)) (only parsing) : order_scope.
Notation "x >^l y" := (y <^l x) (only parsing) : order_scope.
Notation "x >^l y :> T" := ((x : T) >^l (y : T)) (only parsing) : order_scope.

Notation "x <=^l y <=^l z" := ((x <=^l y) && (y <=^l z)) : order_scope.
Notation "x <^l y <=^l z" := ((x <^l y) && (y <=^l z)) : order_scope.
Notation "x <=^l y <^l z" := ((x <=^l y) && (y <^l z)) : order_scope.
Notation "x <^l y <^l z" := ((x <^l y) && (y <^l z)) : order_scope.

Notation "x <=^l y ?= 'iff' C" := (<?=^l%O x y C) : order_scope.
Notation "x <=^l y ?= 'iff' C :> T" := ((x : T) <=^l (y : T) ?= iff C)
  (only parsing) : order_scope.

Notation ">=<^l y" := [pred x | >=<^l%O x y] : order_scope.
Notation ">=<^l y :> T" := (>=<^l (y : T)) (only parsing) : order_scope.
Notation "x >=<^l y" := (>=<^l%O x y) : order_scope.

Notation "><^l y" := [pred x | ~~ (>=<^l%O x y)] : order_scope.
Notation "><^l y :> T" := (><^l (y : T)) (only parsing) : order_scope.
Notation "x ><^l y" := (~~ (><^l%O x y)) : order_scope.

Notation meetlexi := (@meet lexi_display _).
Notation joinlexi := (@join lexi_display _).

Notation "x `&^l` y" := (meetlexi x y) : order_scope.
Notation "x `|^l` y" := (joinlexi x y) : order_scope.

End LexiSyntax.

We declare a "copy" of the cartesian product which has canonical product order.

Module ProdOrder.
Section ProdOrder.

Local Open Scope type_scope. (* FIXME *)

Definition type (disp : unit) (T T' : Type) := T × T'.

Context {disp1 disp2 disp3 : unit}.


#[export] HB.instance Definition _ (T T' : eqType) := Equality.on (T × T').
#[export] HB.instance Definition _ (T T' : choiceType) := Choice.on (T × T').
#[export] HB.instance Definition _ (T T' : countType) := Countable.on (T × T').
#[export] HB.instance Definition _ (T T' : finType) := Finite.on (T × T').

Section POrder.
Variable (T : porderType disp1) (T' : porderType disp2).

Implicit Types (x y : T × T').

Definition le x y := (x.1 y.1) && (x.2 y.2).

Fact refl : reflexive le.

Fact anti : antisymmetric le.

Fact trans : transitive le.

#[export]
HB.instance Definition _ :=
  isPOrder.Build disp3 (T × T') (rrefl _) refl anti trans.

Lemma leEprod x y : (x y) = (x.1 y.1) && (x.2 y.2).

Lemma ltEprod x y : (x < y) = [&& x != y, x.1 y.1 & x.2 y.2].

Lemma le_pair (x1 y1 : T) (x2 y2 : T') :
  (x1, x2) (y1, y2) :> T × T' = (x1 y1) && (x2 y2).

Lemma lt_pair (x1 y1 : T) (x2 y2 : T') : (x1, x2) < (y1, y2) :> T × T' =
  [&& (x1 != y1) || (x2 != y2), x1 y1 & x2 y2].

End POrder.

Section Lattice.
Variable (T : latticeType disp1) (T' : latticeType disp2).
Implicit Types (x y : T × T').

Definition meet x y := (x.1 `&` y.1, x.2 `&` y.2).
Definition join x y := (x.1 `|` y.1, x.2 `|` y.2).

Fact meetC : commutative meet.

Fact joinC : commutative join.

Fact meetA : associative meet.

Fact joinA : associative join.

Fact joinKI y x : meet x (join x y) = x.

Fact meetKU y x : join x (meet x y) = x.

Fact leEmeet x y : (x y) = (meet x y == x).

#[export]
HB.instance Definition _ := POrder_isLattice.Build
  _ (T × T') meetC joinC meetA joinA joinKI meetKU leEmeet.

Lemma meetEprod x y : x `&` y = (x.1 `&` y.1, x.2 `&` y.2).

Lemma joinEprod x y : x `|` y = (x.1 `|` y.1, x.2 `|` y.2).

End Lattice.

Section BLattice.
Variable (T : bLatticeType disp1) (T' : bLatticeType disp2).

Fact le0x (x : T × T') : (\bot, \bot) x :> T × T'.

#[export]
HB.instance Definition _ := hasBottom.Build _ (T × T') le0x.

Lemma botEprod : \bot = (\bot, \bot) :> T × T'.

End BLattice.

Section TBLattice.
Variable (T : tbLatticeType disp1) (T' : tbLatticeType disp2).

Fact lex1 (x : T × T') : x (top, top).

#[export]
HB.instance Definition _ := hasTop.Build _ (T × T') lex1.

Lemma topEprod : \top = (\top, \top) :> T × T'.

End TBLattice.

Section DistrLattice.
Variable (T : distrLatticeType disp1) (T' : distrLatticeType disp2).

Fact meetUl : left_distributive (@meet T T') (@join T T').

#[export]
HB.instance Definition _ := Lattice_Meet_isDistrLattice.Build _ (T × T') meetUl.

End DistrLattice.

FIXME: the canonical (t)bDistrLatticeType instances of products should be automatically generated.
#[export]
HB.instance Definition _
  (T : bDistrLatticeType disp1) (T' : bDistrLatticeType disp2) :=
  DistrLattice.on (T × T').

#[export]
HB.instance Definition _
  (T : tbDistrLatticeType disp1) (T' : tbDistrLatticeType disp2) :=
  DistrLattice.on (T × T').
/FIXME

Section CBDistrLattice.
Variable (T : cbDistrLatticeType disp1) (T' : cbDistrLatticeType disp2).
Implicit Types (x y : T × T').

Definition diff x y := (x.1 `\` y.1, x.2 `\` y.2).

Lemma diffKI x y : y `&` diff x y = \bot.

Lemma joinIB x y : x `&` y `|` diff x y = x.

#[export]
HB.instance Definition _ := hasRelativeComplement.Build _ (T × T') diffKI joinIB.

Lemma subEprod x y : x `\` y = (x.1 `\` y.1, x.2 `\` y.2).

End CBDistrLattice.

Section CTBDistrLattice.
Variable (T : ctbDistrLatticeType disp1) (T' : ctbDistrLatticeType disp2).
Implicit Types (x y : T × T').

Definition compl x : T × T' := (~` x.1, ~` x.2).

Lemma complE x : compl x = diff \top x.

#[export]
HB.instance Definition _ := hasComplement.Build _ (T × T') complE.

Lemma complEprod x : ~` x = (~` x.1, ~` x.2).

End CTBDistrLattice.

FIXME
#[export]
HB.instance Definition _ (T : finPOrderType disp1)
  (T' : finPOrderType disp2) := POrder.on (T × T').
#[export]
HB.instance Definition _ (T : finLatticeType disp1)
  (T' : finLatticeType disp2) := Lattice.on (T × T').
#[export]
HB.instance Definition _ (T : finDistrLatticeType disp1)
  (T' : finDistrLatticeType disp2) := DistrLattice.on (T × T').
#[export]
HB.instance Definition _ (T : finCDistrLatticeType disp1)
  (T' : finCDistrLatticeType disp2) := CTBDistrLattice.on (T × T').
/FIXME

End ProdOrder.

Module Exports.
Notation "T *prod[ d ] T'" := (type d T T')
  (at level 70, d at next level, format "T *prod[ d ] T'") : type_scope.
Notation "T *p T'" := (type prod_display T T')
  (at level 70, format "T *p T'") : type_scope.
Definition leEprod := @leEprod.
Definition ltEprod := @ltEprod.
Definition le_pair := @le_pair.
Definition lt_pair := @lt_pair.
Definition meetEprod := @meetEprod.
Definition joinEprod := @joinEprod.
Definition botEprod := @botEprod.
Definition topEprod := @topEprod.
Definition subEprod := @subEprod.
Definition complEprod := @complEprod.
End Exports.
End ProdOrder.

Module DefaultProdOrder.
Section DefaultProdOrder.
Context {disp1 disp2 : unit}.

FIXME: Scopes of arguments are broken in several places. FIXME: Declaring a bunch of copies is still a bit painful.
We declare lexicographic ordering on dependent pairs.

Module SigmaOrder.
Section SigmaOrder.

Context {disp1 disp2 : unit}.

Section POrder.

Variable (T : porderType disp1) (T' : T porderType disp2).
Implicit Types (x y : {t : T & T' t}).

Definition le x y := (tag x tag y) &&
  ((tag x tag y) ==> (tagged x tagged_as x y)).
Definition lt x y := (tag x tag y) &&
  ((tag x tag y) ==> (tagged x < tagged_as x y)).

Fact refl : reflexive le.

Fact anti : antisymmetric le.

Fact trans : transitive le.

Fact lt_def x y : lt x y = (y != x) && le x y.

#[export]
HB.instance Definition _ :=
  isPOrder.Build disp2 {t : T & T' t} lt_def refl anti trans.

Lemma leEsig x y : x y =
  (tag x tag y) && ((tag x tag y) ==> (tagged x tagged_as x y)).

Lemma ltEsig x y : x < y =
  (tag x tag y) && ((tag x tag y) ==> (tagged x < tagged_as x y)).

Lemma le_Taggedl x (u : T' (tag x)) : (Tagged T' u x) = (u tagged x).

Lemma le_Taggedr x (u : T' (tag x)) : (x Tagged T' u) = (tagged x u).

Lemma lt_Taggedl x (u : T' (tag x)) : (Tagged T' u < x) = (u < tagged x).

Lemma lt_Taggedr x (u : T' (tag x)) : (x < Tagged T' u) = (tagged x < u).

End POrder.

FIXME
#[export]
HB.instance Definition _ (T : finPOrderType disp1)
  (T' : T finPOrderType disp2) := POrder.on {t : T & T' t}.
/FIXME

Section Total.
Variable (T : orderType disp1) (T' : T orderType disp2).
Implicit Types (x y : {t : T & T' t}).

Fact total : total (<=%O : rel {t : T & T' t}).

#[export]
HB.instance Definition _ := POrder_isTotal.Build _ {t : T & T' t} total.

End Total.

Section FinDistrLattice.
Variable (T : finOrderType disp1) (T' : T finOrderType disp2).

Fact le0x (x : {t : T & T' t}) : Tagged T' (\bot : T' \bot) x.
#[export]
HB.instance Definition _ := hasBottom.Build _ {t : T & T' t} le0x.

Lemma botEsig : \bot = Tagged T' (\bot : T' \bot).

Fact lex1 (x : {t : T & T' t}) : x Tagged T' (\top : T' \top).
#[export]
HB.instance Definition _ := hasTop.Build _ {t : T & T' t} lex1.

Lemma topEsig : \top = Tagged T' (\top : T' \top).

End FinDistrLattice.

End SigmaOrder.

Module Exports.
Definition leEsig := @leEsig.
Definition ltEsig := @ltEsig.
Definition le_Taggedl := @le_Taggedl.
Definition lt_Taggedl := @lt_Taggedl.
Definition le_Taggedr := @le_Taggedr.
Definition lt_Taggedr := @lt_Taggedr.
Definition topEsig := @topEsig.
Definition botEsig := @botEsig.
End Exports.
End SigmaOrder.

We declare a "copy" of the cartesian product, which has canonical lexicographic order.

Module ProdLexiOrder.
Section ProdLexiOrder.

Local Open Scope type_scope. (* FIXME *)

Definition type (disp : unit) (T T' : Type) := T × T'.

Context {disp1 disp2 disp3 : unit}.


#[export] HB.instance Definition _ (T T' : eqType) := Equality.on (T × T').
#[export] HB.instance Definition _ (T T' : choiceType) := Choice.on (T × T').
#[export] HB.instance Definition _ (T T' : countType) := Countable.on (T × T').
#[export] HB.instance Definition _ (T T' : finType) := Finite.on (T × T').

Section POrder.
Variable (T : porderType disp1) (T' : porderType disp2).

Implicit Types (x y : T × T').

Definition le x y := (x.1 y.1) && ((x.1 y.1) ==> (x.2 y.2)).
Definition lt x y := (x.1 y.1) && ((x.1 y.1) ==> (x.2 < y.2)).

Fact refl : reflexive le.

Fact anti : antisymmetric le.

Fact trans : transitive le.

Fact lt_def x y : lt x y = (y != x) && le x y.

#[export]
HB.instance Definition _ :=
  isPOrder.Build disp3 (T × T') lt_def refl anti trans.

Lemma leEprodlexi x y :
  (x y) = (x.1 y.1) && ((x.1 y.1) ==> (x.2 y.2)).

Lemma ltEprodlexi x y :
  (x < y) = (x.1 y.1) && ((x.1 y.1) ==> (x.2 < y.2)).

Lemma lexi_pair (x1 y1 : T) (x2 y2 : T') :
   (x1, x2) (y1, y2) :> T × T' = (x1 y1) && ((x1 y1) ==> (x2 y2)).

Lemma ltxi_pair (x1 y1 : T) (x2 y2 : T') :
   (x1, x2) < (y1, y2) :> T × T' = (x1 y1) && ((x1 y1) ==> (x2 < y2)).

End POrder.

FIXME
#[export]
HB.instance Definition _ (T : finPOrderType disp1)
  (T' : finPOrderType disp2) := POrder.on (T × T').
/FIXME

Section Total.
Variable (T : orderType disp1) (T' : orderType disp2).
Implicit Types (x y : T × T').

Fact total : total (<=%O : rel (T × T')).

#[export]
HB.instance Definition _ := POrder_isTotal.Build _ (T × T') total.

End Total.

Section FinDistrLattice.
Variable (T : finOrderType disp1) (T' : finOrderType disp2).

Fact le0x (x : T × T') : (\bot, \bot) x :> T × T'.

#[export]
HB.instance Definition _ := hasBottom.Build _ (T × T') le0x.

Lemma botEprodlexi : \bot = (\bot, \bot) :> T × T'.

Fact lex1 (x : T × T') : x (\top, \top) :> T × T'.

#[export]
HB.instance Definition _ := hasTop.Build _ (T × T') lex1.

Lemma topEprodlexi : \top = (\top, \top) :> T × T'.

End FinDistrLattice.

Lemma sub_prod_lexi d (T : porderType disp1) (T' : porderType disp2) :
   subrel (<=%O : rel (T ×prod[d] T')) (<=%O : rel (T × T')).

End ProdLexiOrder.

Module Exports.


Notation "T *lexi[ d ] T'" := (type d T T')
  (at level 70, d at next level, format "T *lexi[ d ] T'") : type_scope.
Notation "T *l T'" := (type lexi_display T T')
  (at level 70, format "T *l T'") : type_scope.

Definition leEprodlexi := @leEprodlexi.
Definition ltEprodlexi := @ltEprodlexi.
Definition lexi_pair := @lexi_pair.
Definition ltxi_pair := @ltxi_pair.
Definition topEprodlexi := @topEprodlexi.
Definition botEprodlexi := @botEprodlexi.
Definition sub_prod_lexi := @sub_prod_lexi.

End Exports.
End ProdLexiOrder.

Module DefaultProdLexiOrder.
Section DefaultProdLexiOrder.
Context {disp1 disp2 : unit}.


End DefaultProdLexiOrder.
End DefaultProdLexiOrder.

We declare a "copy" of the sequences, which has canonical product order.

Module SeqProdOrder.
Section SeqProdOrder.

Definition type (disp : unit) T := seq T.

Context {disp disp' : unit}.


#[export] HB.instance Definition _ (T : eqType) := Equality.on (seq T).
#[export] HB.instance Definition _ (T : choiceType) := Choice.on (seq T).
#[export] HB.instance Definition _ (T : countType) := Countable.on (seq T).

Section POrder.
Variable T : porderType disp.
Implicit Types s : seq T.

Fixpoint le s1 s2 := if s1 isn't x1 :: s1' then true else
                     if s2 isn't x2 :: s2' then false else
                     (x1 x2) && le s1' s2'.

Fact refl : reflexive le.

Fact anti : antisymmetric le.

Fact trans : transitive le.

#[export]
HB.instance Definition _ := isPOrder.Build disp' (seq T) (rrefl _) refl anti trans.

Lemma leEseq s1 s2 : s1 s2 = if s1 isn't x1 :: s1' then true else
                                if s2 isn't x2 :: s2' then false else
                                (x1 x2) && (s1' s2' :> seq _).

Lemma le0s s : [::] s :> seq _.

Lemma les0 s : s [::] = (s == [::]).

Lemma le_cons x1 s1 x2 s2 :
   x1 :: s1 x2 :: s2 :> seq _ = (x1 x2) && (s1 s2).

End POrder.

Section Lattice.
Variable T : latticeType disp.
Implicit Types s : seq T.

Fixpoint meet s1 s2 :=
  match s1, s2 with
    | x1 :: s1', x2 :: s2'(x1 `&` x2) :: meet s1' s2'
    | _, _[::]
  end.

Fixpoint join s1 s2 :=
  match s1, s2 with
    | [::], _s2 | _, [::]s1
    | x1 :: s1', x2 :: s2'(x1 `|` x2) :: join s1' s2'
  end.

Fact meetC : commutative meet.

Fact joinC : commutative join.

Fact meetA : associative meet.

Fact joinA : associative join.

Fact meetss s : meet s s = s.

Fact joinKI y x : meet x (join x y) = x.

Fact meetKU y x : join x (meet x y) = x.

Fact leEmeet x y : (x y) = (meet x y == x).

#[export]
HB.instance Definition _ :=
  POrder_isLattice.Build _ (seq T) meetC joinC meetA joinA joinKI meetKU leEmeet.

Lemma meetEseq s1 s2 : s1 `&` s2 = [seq x.1 `&` x.2 | x <- zip s1 s2].

Lemma meet_cons x1 s1 x2 s2 :
  (x1 :: s1 : seq T) `&` (x2 :: s2) = (x1 `&` x2) :: s1 `&` s2.

Lemma joinEseq s1 s2 : s1 `|` s2 =
  match s1, s2 with
    | [::], _s2 | _, [::]s1
    | x1 :: s1', x2 :: s2'(x1 `|` x2) :: ((s1' : seq _) `|` s2')
  end.

Lemma join_cons x1 s1 x2 s2 :
  (x1 :: s1 : seq T) `|` (x2 :: s2) = (x1 `|` x2) :: s1 `|` s2.

#[export]
HB.instance Definition _ := hasBottom.Build _ (seq T) (@le0s _).

Lemma botEseq : \bot = [::] :> seq T.

End Lattice.

Section DistrLattice.
Variable T : distrLatticeType disp.

Fact meetUl : left_distributive (@meet T) (@join T).

#[export]
HB.instance Definition _ :=
  Lattice_Meet_isDistrLattice.Build _ (seq T) meetUl.

End DistrLattice.

End SeqProdOrder.

Module Exports.


Notation seqprod_with := type.
Notation seqprod := (type prod_display).

Definition leEseq := @leEseq.
Definition le0s := @le0s.
Definition les0 := @les0.
Definition le_cons := @le_cons.
Definition botEseq := @botEseq.
Definition meetEseq := @meetEseq.
Definition meet_cons := @meet_cons.
Definition joinEseq := @joinEseq.

End Exports.
End SeqProdOrder.

Module DefaultSeqProdOrder.
Section DefaultSeqProdOrder.
Context {disp : unit}.


End DefaultSeqProdOrder.
End DefaultSeqProdOrder.

We declare a "copy" of the sequences, which has canonical lexicographic order.

Module SeqLexiOrder.
Section SeqLexiOrder.

Definition type (disp : unit) T := seq T.

Context {disp disp' : unit}.


#[export] HB.instance Definition _ (T : eqType) := Equality.on (seq T).
#[export] HB.instance Definition _ (T : choiceType) := Choice.on (seq T).
#[export] HB.instance Definition _ (T : countType) := Countable.on (seq T).

Section POrder.
Variable T : porderType disp.
Implicit Types s : seq T.

Fixpoint le s1 s2 := if s1 isn't x1 :: s1' then true else
                     if s2 isn't x2 :: s2' then false else
                       (x1 x2) && ((x1 x2) ==> le s1' s2').
Fixpoint lt s1 s2 := if s2 isn't x2 :: s2' then false else
                     if s1 isn't x1 :: s1' then true else
                       (x1 x2) && ((x1 x2) ==> lt s1' s2').

Fact refl: reflexive le.

Fact anti: antisymmetric le.

Fact trans: transitive le.

Lemma lt_def s1 s2 : lt s1 s2 = (s2 != s1) && le s1 s2.

#[export]
HB.instance Definition _ := isPOrder.Build disp' (seq T) lt_def refl anti trans.

Lemma leEseqlexi s1 s2 :
   s1 s2 = if s1 isn't x1 :: s1' then true else
              if s2 isn't x2 :: s2' then false else
              (x1 x2) && ((x1 x2) ==> (s1' s2' :> seq T)).

Lemma ltEseqlexi s1 s2 :
   s1 < s2 = if s2 isn't x2 :: s2' then false else
              if s1 isn't x1 :: s1' then true else
              (x1 x2) && ((x1 x2) ==> (s1' < s2' :> seq T)).

Lemma lexi0s s : [::] s :> seq T.

Lemma lexis0 s : s [::] = (s == [::]).

Lemma ltxi0s s : ([::] < s :> seq T) = (s != [::]).

Lemma ltxis0 s : s < [::] = false.

Lemma lexi_cons x1 s1 x2 s2 :
  x1 :: s1 x2 :: s2 :> seq T = (x1 x2) && ((x1 x2) ==> (s1 s2)).

Lemma ltxi_cons x1 s1 x2 s2 :
  x1 :: s1 < x2 :: s2 :> seq T = (x1 x2) && ((x1 x2) ==> (s1 < s2)).

Lemma lexi_lehead x s1 y s2 : x :: s1 y :: s2 :> seq T x y.

Lemma ltxi_lehead x s1 y s2 : x :: s1 < y :: s2 :> seq T x y.

Lemma eqhead_lexiE (x : T) s1 s2 : (x :: s1 x :: s2 :> seq _) = (s1 s2).

Lemma eqhead_ltxiE (x : T) s1 s2 : (x :: s1 < x :: s2 :> seq _) = (s1 < s2).

Lemma neqhead_lexiE (x y : T) s1 s2 : x != y
  (x :: s1 y :: s2 :> seq _) = (x < y).

Lemma neqhead_ltxiE (x y : T) s1 s2 : x != y
  (x :: s1 < y :: s2 :> seq _) = (x < y).

End POrder.

Section Total.
Variable T : orderType disp.
Implicit Types s : seq T.

Fact total : total (<=%O : rel (seq T)).

#[export]
HB.instance Definition _ := POrder_isTotal.Build _ (seq T) total.
#[export]
HB.instance Definition _ := hasBottom.Build _ (seq T) (@lexi0s _).

End Total.

Lemma sub_seqprod_lexi d (T : porderType disp) :
   subrel (<=%O : rel (seqprod_with d T)) (<=%O : rel (seq T)).

End SeqLexiOrder.

Module Exports.


Notation seqlexi_with := type.
Notation seqlexi := (type lexi_display).

Definition leEseqlexi := @leEseqlexi.
Definition lexi0s := @lexi0s.
Definition lexis0 := @lexis0.
Definition lexi_cons := @lexi_cons.
Definition lexi_lehead := @lexi_lehead.
Definition eqhead_lexiE := @eqhead_lexiE.
Definition neqhead_lexiE := @neqhead_lexiE.

Definition ltEseqltxi := @ltEseqlexi.
Definition ltxi0s := @ltxi0s.
Definition ltxis0 := @ltxis0.
Definition ltxi_cons := @ltxi_cons.
Definition ltxi_lehead := @ltxi_lehead.
Definition eqhead_ltxiE := @eqhead_ltxiE.
Definition neqhead_ltxiE := @neqhead_ltxiE.
Definition sub_seqprod_lexi := @sub_seqprod_lexi.

End Exports.
End SeqLexiOrder.

Module DefaultSeqLexiOrder.
Section DefaultSeqLexiOrder.
Context {disp : unit}.


End DefaultSeqLexiOrder.
End DefaultSeqLexiOrder.

We declare a "copy" of the tuples, which has canonical product order.

Module TupleProdOrder.
Import DefaultSeqProdOrder.

Section TupleProdOrder.

Definition type (disp : unit) n T := n.-tuple T.

Context {disp disp' : unit}.

Section Basics.
Variable (n : nat).
#[export] HB.instance Definition _ (T : eqType) := Equality.on (n.-tuple T).
#[export] HB.instance Definition _ (T : choiceType) := Choice.on (n.-tuple T).
#[export] HB.instance Definition _ (T : countType) := Countable.on (n.-tuple T).
#[export] HB.instance Definition _ (T : finType) := Finite.on (n.-tuple T).
End Basics.

Section POrder.
Implicit Types (T : porderType disp).

#[export] HB.instance Definition _ n T := SubChoice.on (n.-tuple T).
#[export] HB.instance Definition _ n T :=
  [SubChoice_isSubPOrder of n.-tuple T by <: with disp'].

Lemma leEtprod n T (t1 t2 : n.-tuple T) :
   t1 t2 = [ i, tnth t1 i tnth t2 i].

Lemma ltEtprod n T (t1 t2 : n.-tuple T) :
  t1 < t2 = [ i, tnth t1 i != tnth t2 i] &&
            [ i, tnth t1 i tnth t2 i].

End POrder.

Section Lattice.
Variables (n : nat) (T : latticeType disp).
Implicit Types (t : n.-tuple T).

Definition meet t1 t2 : n.-tuple T :=
  [tuple of [seq x.1 `&` x.2 | x <- zip t1 t2]].
Definition join t1 t2 : n.-tuple T :=
  [tuple of [seq x.1 `|` x.2 | x <- zip t1 t2]].

Fact tnth_meet t1 t2 i : tnth (meet t1 t2) i = tnth t1 i `&` tnth t2 i.

Fact tnth_join t1 t2 i : tnth (join t1 t2) i = tnth t1 i `|` tnth t2 i.

Fact meetC : commutative meet.

Fact joinC : commutative join.

Fact meetA : associative meet.

Fact joinA : associative join.

Fact joinKI t2 t1 : meet t1 (join t1 t2) = t1.

Fact meetKU y x : join x (meet x y) = x.

Fact leEmeet t1 t2 : (t1 t2) = (meet t1 t2 == t1).

#[export]
HB.instance Definition _ := POrder_isLattice.Build
  _ (n.-tuple T) meetC joinC meetA joinA joinKI meetKU leEmeet.

Lemma meetEtprod t1 t2 :
  t1 `&` t2 = [tuple of [seq x.1 `&` x.2 | x <- zip t1 t2]].

Lemma joinEtprod t1 t2 :
  t1 `|` t2 = [tuple of [seq x.1 `|` x.2 | x <- zip t1 t2]].

End Lattice.

Section BLattice.
Variables (n : nat) (T : bLatticeType disp).
Implicit Types (t : n.-tuple T).

Fact le0x t : [tuple of nseq n \bot] t :> n.-tuple T.

#[export]
HB.instance Definition _ := hasBottom.Build _ (n.-tuple T) le0x.

Lemma botEtprod : \bot = [tuple of nseq n \bot] :> n.-tuple T.

End BLattice.

Section TBLattice.
Variables (n : nat) (T : tbLatticeType disp).
Implicit Types (t : n.-tuple T).

Fact lex1 t : t [tuple of nseq n \top] :> n.-tuple T.

#[export]
HB.instance Definition _ := hasTop.Build _ (n.-tuple T) lex1.

Lemma topEtprod : \top = [tuple of nseq n \top] :> n.-tuple T.

End TBLattice.

Section DistrLattice.
Variables (n : nat) (T : distrLatticeType disp).
Implicit Types (t : n.-tuple T).

Fact meetUl : left_distributive (@meet n T) (@join n T).

#[export]
HB.instance Definition _ :=
  Lattice_Meet_isDistrLattice.Build _ (n.-tuple T) meetUl.

End DistrLattice.

FIXME
#[export]
HB.instance Definition _ (n : nat) (T : bDistrLatticeType disp) :=
  DistrLattice.on (n.-tuple T).
#[export]
HB.instance Definition _ (n : nat) (T : tbDistrLatticeType disp) :=
  DistrLattice.on (n.-tuple T).
/FIXME

Section CBDistrLattice.
Variables (n : nat) (T : cbDistrLatticeType disp).
Implicit Types (t : n.-tuple T).

Definition diff t1 t2 : n.-tuple T :=
  [tuple of [seq x.1 `\` x.2 | x <- zip t1 t2]].

Fact tnth_diff t1 t2 i : tnth (diff t1 t2) i = tnth t1 i `\` tnth t2 i.
#[deprecated(since="mathcomp 2.0.0", note="Use tnth_diff instead.")]
Notation tnth_sub := tnth_diff.

Lemma diffKI t1 t2 : t2 `&` diff t1 t2 = \bot.

Lemma joinIB t1 t2 : t1 `&` t2 `|` diff t1 t2 = t1.

#[export] HB.instance Definition _ := hasRelativeComplement.Build _ (n.-tuple T) diffKI joinIB.

Lemma diffEtprod t1 t2 :
  t1 `\` t2 = [tuple of [seq x.1 `\` x.2 | x <- zip t1 t2]].
#[deprecated(since="mathcomp 2.0.0", note="Use diffEtprod instead.")]
Notation subEtprod := diffEtprod.

End CBDistrLattice.

Section CTBDistrLattice.
Variables (n : nat) (T : ctbDistrLatticeType disp).
Implicit Types (t : n.-tuple T).

Definition compl t : n.-tuple T := map_tuple compl t.

Fact tnth_compl t i : tnth (compl t) i = ~` tnth t i.

Lemma complE t : compl t = diff \top t.

#[export] HB.instance Definition _ := hasComplement.Build _ (n.-tuple T) complE.

Lemma complEtprod t : ~` t = [tuple of [seq ~` x | x <- t]].

End CTBDistrLattice.

FIXME
#[export]
HB.instance Definition _ (n : nat) (T : finPOrderType disp) :=
  POrder.on (n.-tuple T).
#[export]
HB.instance Definition _ (n : nat) (T : finLatticeType disp) :=
  Lattice.on (n.-tuple T).
#[export]
HB.instance Definition _ (n : nat) (T : finDistrLatticeType disp) :=
  DistrLattice.on (n.-tuple T).
#[export]
HB.instance Definition _ (n : nat) (T : finCDistrLatticeType disp) :=
  CTBDistrLattice.on (n.-tuple T).
/FIXME

End TupleProdOrder.

Module Exports.


Notation "n .-tupleprod[ disp ]" := (type disp n)
  (at level 2, disp at next level, format "n .-tupleprod[ disp ]") :
  type_scope.
Notation "n .-tupleprod" := (n.-tupleprod[prod_display])
  (at level 2, format "n .-tupleprod") : type_scope.

Definition leEtprod := @leEtprod.
Definition ltEtprod := @ltEtprod.
Definition meetEtprod := @meetEtprod.
Definition joinEtprod := @joinEtprod.
Definition botEtprod := @botEtprod.
Definition topEtprod := @topEtprod.
Definition diffEtprod := @diffEtprod.
Definition complEtprod := @complEtprod.

Definition tnth_meet := @tnth_meet.
Definition tnth_join := @tnth_join.
Definition tnth_diff := @tnth_diff.
Definition tnth_compl := @tnth_compl.

End Exports.
End TupleProdOrder.

Module DefaultTupleProdOrder.
Section DefaultTupleProdOrder.
Context {disp : unit}.


End DefaultTupleProdOrder.
End DefaultTupleProdOrder.

We declare a "copy" of the tuples, which has canonical lexicographic order.

Module TupleLexiOrder.
Section TupleLexiOrder.
Import DefaultSeqLexiOrder.

Definition type (disp : unit) n T := n.-tuple T.

Context {disp disp' : unit}.

Section Basics.
Variable (n : nat).
#[export] HB.instance Definition _ (T : eqType) := Equality.on (n.-tuple T).
#[export] HB.instance Definition _ (T : choiceType) := Choice.on (n.-tuple T).
#[export] HB.instance Definition _ (T : countType) := Countable.on (n.-tuple T).
#[export] HB.instance Definition _ (T : finType) := Finite.on (n.-tuple T).
End Basics.

Section POrder.
Implicit Types (T : porderType disp).

#[export] HB.instance Definition _ n T := SubChoice.on (n.-tuple T).
#[export] HB.instance Definition _ n T :=
  [SubChoice_isSubPOrder of n.-tuple T by <: with disp'].

Lemma lexi_tupleP n T (t1 t2 : n.-tuple T) :
   reflect ( k : 'I_n.+1, i : 'I_n, (i k)%N
               tnth t1 i tnth t2 i ?= iff (i != k :> nat)) (t1 t2).

Lemma ltxi_tupleP n T (t1 t2 : n.-tuple T) :
   reflect ( k : 'I_n, i : 'I_n, (i k)%N
               tnth t1 i tnth t2 i ?= iff (i != k :> nat)) (t1 < t2).

Lemma ltxi_tuplePlt n T (t1 t2 : n.-tuple T) : reflect
  (exists2 k : 'I_n, i : 'I_n, (i < k)%N tnth t1 i = tnth t2 i
                                                 & tnth t1 k < tnth t2 k)
  (t1 < t2).

End POrder.

FIXME
#[export]
HB.instance Definition _ (n : nat) (T : finPOrderType disp) :=
  POrder.on (n.-tuple T).
/FIXME

#[export] HB.instance Definition _ n (T : orderType disp) :=
  SubChoice.on (n.-tuple T).
#[export] HB.instance Definition _ n (T : orderType disp) :=
  [SubChoice_isSubOrder of n.-tuple T by <: with disp'].

Section BDistrLattice.
Variables (n : nat) (T : finOrderType disp).
Implicit Types (t : n.-tuple T).

Fact le0x t : [tuple of nseq n \bot] t :> n.-tuple T.

#[export] HB.instance Definition _ := hasBottom.Build _ (n.-tuple T) le0x.

Lemma botEtlexi : \bot = [tuple of nseq n \bot] :> n.-tuple T.

End BDistrLattice.

Section TBDistrLattice.
Variables (n : nat) (T : finOrderType disp).
Implicit Types (t : n.-tuple T).

Fact lex1 t : t [tuple of nseq n \top].

#[export] HB.instance Definition _ := hasTop.Build _ (n.-tuple T) lex1.

Lemma topEtlexi : \top = [tuple of nseq n \top] :> n.-tuple T.

End TBDistrLattice.

Lemma sub_tprod_lexi d n (T : porderType disp) :
   subrel (<=%O : rel (n.-tupleprod[d] T)) (<=%O : rel (n.-tuple T)).

End TupleLexiOrder.

Module Exports.


Notation "n .-tuplelexi[ disp ]" := (type disp n)
  (at level 2, disp at next level, format "n .-tuplelexi[ disp ]") :
  type_scope.
Notation "n .-tuplelexi" := (n.-tuplelexi[lexi_display])
  (at level 2, format "n .-tuplelexi") : type_scope.

Definition lexi_tupleP := @lexi_tupleP.
Arguments lexi_tupleP {disp disp' n T t1 t2}.
Definition ltxi_tupleP := @ltxi_tupleP.
Arguments ltxi_tupleP {disp disp' n T t1 t2}.
Definition ltxi_tuplePlt := @ltxi_tuplePlt.
Arguments ltxi_tuplePlt {disp disp' n T t1 t2}.
Definition topEtlexi := @topEtlexi.
Definition botEtlexi := @botEtlexi.
Definition sub_tprod_lexi := @sub_tprod_lexi.

End Exports.
End TupleLexiOrder.

Module DefaultTupleLexiOrder.
Section DefaultTupleLexiOrder.
Context {disp : unit}.


End DefaultTupleLexiOrder.
End DefaultTupleLexiOrder.

Module Import DualOrder.
Section DualOrder.
Context {disp : unit}.
Variable O : orderType disp.

Lemma dual_total : total (<=%O : rel O^d).

#[export]
HB.instance Definition _ := DistrLattice_isTotal.Build _ O^d dual_total.

End DualOrder.

#[export]
HB.instance Definition _ d (T : finOrderType d) := FinTotal.on T^d.

Section DualOrderTheory.

Context {disp : unit} {T : orderType disp}.
Implicit Type s : seq T.

Lemma sorted_filter_gt x s :
  sorted <=%O s [seq y <- s | x < y] = drop (count ( x) s) s.

Lemma sorted_filter_ge x s :
  sorted <=%O s [seq y <- s | x y] = drop (count (< x) s) s.

Lemma nth_count_ge x x0 s i : sorted <=%O s
  (count (< x) s i < size s)%N x nth x0 s i.

Lemma nth_count_gt x x0 s i : sorted <=%O s
  (count ( x) s i < size s)%N x < nth x0 s i.

Lemma nth_count_eq x x0 s i : sorted <=%O s
  (count (< x) s i < count ( x) s)%N nth x0 s i = x.

End DualOrderTheory.

End DualOrder.

We declare a "copy" of the sets, which is canonically ordered by inclusion

Module SetSubsetOrder.
Section SetSubsetOrder.

Definition type (disp : unit) (T : finType) := {set T}.

Context {disp : unit} {T : finType}.
Implicit Type (A B C : {subset T}).

Lemma le_def A B : A \subset B = (A :&: B == A).

Lemma setKUC B A : A :&: (A :|: B) = A.

Lemma setKIC B A : A :|: (A :&: B) = A.

#[export]
HB.instance Definition _ := Choice.on {subset T}.

#[export]
HB.instance Definition _ := isMeetJoinDistrLattice.Build disp {subset T}
  le_def (fun _ _erefl) (@setIC _) (@setUC _) (@setIA _) (@setUA _)
  setKUC setKIC (@setIUl _) (@setIid _).

#[export]
HB.instance Definition _ := hasBottom.Build disp {subset T} (@sub0set _).

#[export]
HB.instance Definition _ := hasTop.Build disp {subset T} (@subsetT _).

Lemma setIDv A B : B :&: (A :\: B) = set0.

#[export]
HB.instance Definition _ := hasRelativeComplement.Build disp {subset T} setIDv (@setID _).

Lemma setTDsym A : ~: A = setT :\: A.

#[export]
HB.instance Definition _ := hasComplement.Build disp {subset T} setTDsym.

Lemma leEsubset A B : (A B) = (A \subset B).
Lemma meetEsubset A B : A `&` B = A :&: B.
Lemma joinEsubset A B : A `|` B = A :|: B.
Lemma botEsubset : \bot = set0 :> {subset T}.
Lemma topEsubset : \top = setT :> {subset T}.
Lemma subEsubset A B : A `\` B = A :\: B.
Lemma complEsubset A : ~` A = ~: A.

Fact subset_display : unit.

End SetSubsetOrder.

Module Exports.
Arguments type disp T%type.
Notation "{ 'subset' [ d ] T }" := (type d T)
  (at level 2, d at next level, format "{ 'subset' [ d ] T }") : type_scope.
Notation "{ 'subset' T }" := {subset[subset_display] T}
  (at level 2, format "{ 'subset' T }") : type_scope.


Definition leEsubset := @leEsubset.
Definition meetEsubset := @meetEsubset.
Definition joinEsubset := @joinEsubset.
Definition botEsubset := @botEsubset.
Definition topEsubset := @topEsubset.
Definition subEsubset := @subEsubset.
Definition complEsubset := @complEsubset.

End Exports.
End SetSubsetOrder.
Export SetSubsetOrder.Exports.

Module DefaultSetSubsetOrder.
Section DefaultSetSubsetOrder.
Context {disp : unit}.


End DefaultSetSubsetOrder.
End DefaultSetSubsetOrder.

Notation enum A := (sort <=%O (enum A)).

Section Enum.
Variables (d : unit) (T : finPOrderType d).

Lemma cardE (A : {pred T}) : #|A| = size (enum A).

Lemma mem_enum (A : {pred T}) : enum A =i A.

Lemma enum_uniq (A : {pred T}) : uniq (enum A).

Lemma cardT : #|T| = size (enum T).

Lemma enumT : enum T = sort <=%O (Finite.enum T).

Lemma enum0 : enum (pred0 : {pred T}) = [::].

Lemma enum1 (x : T) : enum (pred1 x) = [:: x].

Lemma eq_enum (A B : {pred T}) : A =i B enum A = enum B.

Lemma eq_cardT (A : {pred T}) : A =i predT #|A| = size (enum T).

Lemma set_enum (A : {set T}) : [set x in enum A] = A.

Lemma enum_set0 : enum (set0 : {set T}) = [::].

Lemma enum_setT : enum [set: T] = sort <=%O (Finite.enum T).

Lemma enum_set1 (a : T) : enum [set a] = [:: a].

End Enum.

Section Ordinal.
Import OrdinalOrder.Exports.

Lemma enum_ord n : enum 'I_n = fintype.enum 'I_n.

Lemma val_enum_ord n : [seq val i | i <- enum 'I_n] = iota 0 n.

Lemma size_enum_ord n : size (enum 'I_n) = n.

Lemma nth_enum_ord (n : nat) (i0 : 'I_n) (m : nat) :
  (m < n)%N nth i0 (enum 'I_n) m = m :> nat.

Lemma nth_ord_enum (n : nat) (i0 i : 'I_n) : nth i0 (enum 'I_n) i = i.

Lemma index_enum_ord (n : nat) (i : 'I_n) : index i (enum 'I_n) = i.

End Ordinal.

Lemma mono_sorted_enum d d' (T : finPOrderType d)
    (T' : porderType d') (f : T T') :
    total (<=%O : rel T) {mono f : x y / (x y)%O}
  sorted <=%O [seq f x | x <- Order.enum T].

Lemma mono_unique d (T T' : finPOrderType d) (f g : T T') :
    total (<=%O : rel T) (#|T'| #|T|)%N
    {mono f : x y / x y} {mono g : x y / x y}
  f =1 g.

This module should be exported on demand, as in module tagnat below
We circumvent a shortcomming of finOrderType which requires the type to be nonempty and we do not want to rule this out
Hypothesis (leT_total : total (<=%O : rel T)).

Lemma le_enum_val A : {mono @enum_val A : i j / i j}.

Lemma le_enum_rank_in x0 A (Ax0 : x0 \in A) :
  {in A &, {mono enum_rank_in Ax0 : x y / x y}}.

Lemma le_enum_rank : {mono enum_rank : i j / i j}.

End total.
End EnumVal.
Arguments enum_val {d T A}.
Arguments enum_rank {d T}.
End EnumVal.

Notation enum_val := enum_val.
Notation enum_rank_in := enum_rank_in.
Notation enum_rank := enum_rank.
Notation enum_valP := enum_valP.
Notation enum_val_nth := enum_val_nth.
Notation nth_enum_rank_in := nth_enum_rank_in.
Notation nth_enum_rank := nth_enum_rank.
Notation enum_rankK_in := enum_rankK_in.
Notation enum_rankK := enum_rankK.
Notation enum_valK_in := enum_valK_in.
Notation enum_valK := enum_valK.
Notation enum_rank_inj := enum_rank_inj.
Notation enum_val_inj := enum_val_inj.
Notation enum_val_bij_in := enum_val_bij_in.
Notation eq_enum_rank_in := eq_enum_rank_in.
Notation enum_rank_in_inj := enum_rank_in_inj.
Notation enum_rank_bij := enum_rank_bij.
Notation enum_val_bij := enum_val_bij.
Notation le_enum_val := le_enum_val.
Notation le_enum_rank_in := le_enum_rank_in.
Notation le_enum_rank := le_enum_rank.

Module Syntax.
Export POSyntax.
Export LatticeSyntax.
Export BLatticeSyntax.
Export TLatticeSyntax.
Export CBDistrLatticeSyntax.
Export CTBDistrLatticeSyntax.
Export DualSyntax.
Export DvdSyntax.
End Syntax.

Module LTheory.
Export POCoercions.
Export POrderTheory.
Export DualPOrder.

Export DualLattice.
Export LatticeTheoryMeet.
Export LatticeTheoryJoin.
Export DistrLatticeTheory.
Export BLatticeTheory.
Export TLatticeTheory.
Export DualTBLattice.
Export TBLatticeTheory.
Export BDistrLatticeTheory.
Export DualTBDistrLattice.
Export TBDistrLatticeTheory.
Export DualOrder. (* FIXME? *)

Export OrderMorphismTheory.
Export LatticeMorphismTheory.
Export BLatticeMorphismTheory.
Export TLatticeMorphismTheory.

Export ClosedPredicates.
Export LatticePred.

Export SubPOrderTheory.
End LTheory.

Module CTheory.
Export LTheory CBDistrLatticeTheory CTBDistrLatticeTheory.
End CTheory.

Module TTheory.
Export LTheory TotalTheory.
End TTheory.

Module Theory.
Export CTheory TotalTheory.
End Theory.

Module Exports.
End Exports.
End Order.

Export Order.Exports.

Export Order.Syntax.

Export Order.POrder.Exports.
Export Order.FinPOrder.Exports.
Export Order.Lattice.Exports.
Export Order.BLattice.Exports.
Export Order.TBLattice.Exports.
Export Order.FinLattice.Exports.
Export Order.DistrLattice.Exports.
Export Order.BDistrLattice.Exports.
Export Order.TBDistrLattice.Exports.
Export Order.FinDistrLattice.Exports.
Export Order.CBDistrLattice.Exports.
Export Order.CTBDistrLattice.Exports.
Export Order.FinCDistrLattice.Exports.
Export Order.Total.Exports.
Export Order.FinTotal.Exports.

FIXME: check if covered by Order.Exports Export Order.NatOrder.Exports. Export Order.NatMonotonyTheory. Export Order.NatDvd.Exports. Export Order.OrdinalOrder.Exports. Export Order.BoolOrder.Exports. Export Order.ProdOrder.Exports. Export Order.SigmaOrder.Exports. Export Order.ProdLexiOrder.Exports. Export Order.SeqProdOrder.Exports. Export Order.SeqLexiOrder.Exports. Export Order.TupleProdOrder.Exports. Export Order.TupleLexiOrder.Exports.

Module DefaultProdOrder := Order.DefaultProdOrder.
Module DefaultSeqProdOrder := Order.DefaultSeqProdOrder.
Module DefaultTupleProdOrder := Order.DefaultTupleProdOrder.
Module DefaultProdLexiOrder := Order.DefaultProdLexiOrder.
Module DefaultSeqLexiOrder := Order.DefaultSeqLexiOrder.
Module DefaultTupleLexiOrder := Order.DefaultTupleLexiOrder.

Import Order.Theory.

Module tagnat.
Section tagnat.
Import Order.EnumVal.

Context {n : nat} {p_ : 'I_n nat}.


Implicit Types (i : 'I_n) (s : ordsum) (p : T).

Lemma card : #|{: T}| = \sum_i p_ i.

Definition sig : ordsum T := enum_val \o cast_ord (esym card).
Definition rank : T ordsum := cast_ord card \o enum_rank.

Lemma sigK : cancel sig rank.
Lemma sig_inj : injective sig.

Lemma rankK : cancel rank sig.
Lemma rank_inj : injective rank.

Definition sig1 s : 'I_n := tag (sig s).
Definition sig2 s : 'I_(p_ (sig1 s)) := tagged (sig s).
Definition Rank i (j : 'I_(p_ i)) := rank (Tagged _ j).

Lemma sigE12 s : sig s = @Tagged _ (sig1 s) _ (sig2 s).

Lemma rankE p : rank p = @Rank (tag p) (tagged p).

Lemma sig2K s : Rank (sig2 s) = s.

Lemma Rank1K i0 (k : 'I_(p_ i0)) : sig1 (Rank k) = i0.

Lemma Rank2K i0 (k : 'I_(p_ i0)) :
  sig2 (Rank k) = cast_ord (congr1 p_ (esym (Rank1K k))) k.
#[local] Hint Resolve sigK rankK : core.

Lemma rank_bij : bijective rank.
Lemma sig_bij : bijective sig.

Lemma rank_bij_on : {on [pred _ | true], bijective rank}.

Lemma sig_bij_on : {on [pred _ | true], bijective sig}.

Lemma le_sig : {mono sig : i j / i j}.

Lemma le_sig1 : {homo sig1 : i j / i j}.

Lemma le_rank : {mono rank : p q / p q}.

Lemma le_Rank i : {mono @Rank i : j k / j k}.

Lemma lt_sig : {mono sig : i j / i < j}.

Lemma lt_rank : {mono rank : p q / p < q}.

Lemma lt_Rank i : {mono @Rank i : j k / j < k}.

Lemma eq_Rank i i' (j : 'I_(p_ i)) (j': 'I_(p_ i')) :
  (Rank j == Rank j' :> nat) = (i == i') && (j == j' :> nat).

Lemma rankEsum p : rank p = \sum_(i < n | (i < tag p)%N) p_ i + tagged p :> nat.

Lemma RankEsum i j : @Rank i j = \sum_(k < n | (k < i)%N) p_ k + j :> nat.

Lemma rect s : s = \sum_(i < n | (i < sig1 s)%N) p_ i + sig2 s :> nat.

Lemma eqRank (i0 j : nat) (li0 : (i0 < n)%N) (lj : (j < p_ (Ordinal li0))%N) :
  (\sum_(i < n | (i < i0)%N) p_ i) + j = Rank (Ordinal lj) :> nat.

End tagnat.
End tagnat.
Arguments tagnat.Rank {n p_}.