@@ -426,6 +426,8 @@ Record finLattice :=
426426 premeet_closed L^~pl elements &
427427 elements != fset0]}.
428428
429+ (*TODO: separate the conjunction into three separate fields *)
430+
429431Canonical finLattice_subType := Eval hnf in [subType for elements].
430432
431433Definition finLattice_eqMixin := Eval hnf in [eqMixin of finLattice by <:].
@@ -678,6 +680,7 @@ Definition fin_joinMixin := JoinRelMixin finjoinC finjoinA lefinjoin.
678680Local Canonical fin_meetOrder := MeetOrder finle finlt finmeet fin_meetMixin.
679681Local Canonical fin_joinOrder := JoinOrder finle finlt finjoin fin_joinMixin.
680682Local Canonical fin_lattice := [lattice of finle].
683+ (* TODO : are these canonical declarations mandatory ? *)
681684
682685End FinLatticeStructure.
683686Module Exports.
@@ -1363,6 +1366,7 @@ Local Canonical tbJoinOrder := [tbJoinOrder of finle].
13631366Local Canonical bLattice := [bLattice of finle].
13641367Local Canonical tLattice := [tLattice of finle].
13651368Local Canonical tbLattice := [tbLattice of finle].
1369+ (* TODO : are canonical declarations mandatory ? *)
13661370
13671371End FinTBLatticeStructure.
13681372Module Exports.
@@ -1488,7 +1492,8 @@ Lemma coatomP {L} {S : {finLattice L}} {a} : reflect
14881492 ([/\ a \in S, (a <_L \ftop_S) &
14891493 forall x, x \in S -> x <_L \ftop_S -> ~~(a <_L x)])
14901494 (coatom S a).
1491- Proof . apply/(iffP idP).
1495+ Proof .
1496+ apply/(iffP idP).
14921497- by move/atomP.
14931498- move=> ?; exact/atomP.
14941499Qed .
@@ -1783,7 +1788,7 @@ Qed.
17831788
17841789Lemma dual_itv_r L (S : {finLattice L}) a b :
17851790 ([<a; b>]_S)^~s = [< b ; a>]_(S^~s).
1786- Proof . by apply/val_inj/Interval.dual_itv_fset_eq. Qed .
1791+ Proof . by apply/val_inj/Interval.dual_itv_fset_eq. Qed .
17871792
17881793Definition dual_itv :=
17891794 (@dual_itv_r, fun L => @dual_itv_r [preLattice of dual_rel <=:L]).
0 commit comments