]> matita.cs.unibo.it Git - helm.git/blob - helm/software/matita/dama/metric_lattice.ma
62a84090cbc446a6a55a0379b85075a4e9160318
[helm.git] / helm / software / matita / dama / metric_lattice.ma
1 (**************************************************************************)
2 (*       ___                                                              *)
3 (*      ||M||                                                             *)
4 (*      ||A||       A project by Andrea Asperti                           *)
5 (*      ||T||                                                             *)
6 (*      ||I||       Developers:                                           *)
7 (*      ||T||         The HELM team.                                      *)
8 (*      ||A||         http://helm.cs.unibo.it                             *)
9 (*      \   /                                                             *)
10 (*       \ /        This file is distributed under the terms of the       *)
11 (*        v         GNU General Public License Version 2                  *)
12 (*                                                                        *)
13 (**************************************************************************)
14
15 set "baseuri" "cic:/matita/metric_lattice/".
16
17 include "metric_set.ma".
18 include "lattice.ma".
19
20 record mlattice (R : ogroup) : Type ≝ {
21   ml_mset_: metric_set R;
22   ml_lattice:> lattice;
23   ml_with_: ms_carr ? ml_mset_ = ap_carr (l_carr ml_lattice)
24 }.
25
26 lemma ml_mset: ∀R.mlattice R → metric_set R.
27 intros (R ml); apply (mk_metric_set R ml); unfold Type_OF_mlattice;
28 cases (ml_with_ ? ml); simplify;
29 [apply (metric ? (ml_mset_ ? ml));|apply (mpositive ? (ml_mset_ ? ml));
30 |apply (mreflexive ? (ml_mset_ ? ml));|apply (msymmetric ? (ml_mset_ ? ml));
31 |apply (mtineq ? (ml_mset_ ? ml))]
32 qed.
33
34 coercion cic:/matita/metric_lattice/ml_mset.con.