Library CompOptCert.Lattice


Constructions of semi-lattices.

Require Import Coqlib.
Require Import Maps.
Require Import FSets.

Local Unset Elimination Schemes.
Local Unset Case Analysis Schemes.

Signatures of semi-lattices

A semi-lattice is a type t equipped with an equivalence relation eq, a boolean equivalence test beq, a partial order ge, a smallest element bot, and an upper bound operation lub. Note that we do not demand that lub computes the least upper bound.

Module Type SEMILATTICE.

  Parameter t: Type.
  Parameter eq: t t Prop.
  Axiom eq_refl: x, eq x x.
  Axiom eq_sym: x y, eq x y eq y x.
  Axiom eq_trans: x y z, eq x y eq y z eq x z.
  Parameter beq: t t bool.
  Axiom beq_correct: x y, beq x y = true eq x y.
  Parameter ge: t t Prop.
  Axiom ge_refl: x y, eq x y ge x y.
  Axiom ge_trans: x y z, ge x y ge y z ge x z.
  Parameter bot: t.
  Axiom ge_bot: x, ge x bot.
  Parameter lub: t t t.
  Axiom ge_lub_left: x y, ge (lub x y) x.
  Axiom ge_lub_right: x y, ge (lub x y) y.

End SEMILATTICE.

A semi-lattice ``with top'' is similar, but also has a greatest element top.

Module Type SEMILATTICE_WITH_TOP.

  Include SEMILATTICE.
  Parameter top: t.
  Axiom ge_top: x, ge top x.

End SEMILATTICE_WITH_TOP.

Semi-lattice over maps


Set Implicit Arguments.

Given a semi-lattice (without top) L, the following functor implements a semi-lattice structure over finite maps from positive numbers to L.t. The default value for these maps is L.bot. Bottom elements are not smashed.

Module LPMap1(L: SEMILATTICE) <: SEMILATTICE.

Definition t := PTree.t L.t.

Definition get (p: positive) (x: t) : L.t :=
  match x!p with NoneL.bot | Some xx end.

Definition set (p: positive) (v: L.t) (x: t) : t :=
  if L.beq v L.bot
  then PTree.remove p x
  else PTree.set p v x.

Lemma gsspec:
   p v x q,
  L.eq (get q (set p v x)) (if peq q p then v else get q x).
Proof.
  intros. unfold set, get.
  destruct (L.beq v L.bot) eqn:EBOT.
  rewrite PTree.grspec. unfold PTree.elt_eq. destruct (peq q p).
  apply L.eq_sym. apply L.beq_correct; auto.
  apply L.eq_refl.
  rewrite PTree.gsspec. destruct (peq q p); apply L.eq_refl.
Qed.

Definition eq (x y: t) : Prop :=
   p, L.eq (get p x) (get p y).

Lemma eq_refl: x, eq x x.
Proof.
  unfold eq; intros. apply L.eq_refl.
Qed.

Lemma eq_sym: x y, eq x y eq y x.
Proof.
  unfold eq; intros. apply L.eq_sym; auto.
Qed.

Lemma eq_trans: x y z, eq x y eq y z eq x z.
Proof.
  unfold eq; intros. eapply L.eq_trans; eauto.
Qed.

Definition beq (x y: t) : bool := PTree.beq L.beq x y.

Lemma beq_correct: x y, beq x y = true eq x y.
Proof.
  unfold beq; intros; red; intros. unfold get.
  rewrite PTree.beq_correct in H. specialize (H p).
  destruct (x!p); destruct (y!p); intuition.
  apply L.beq_correct; auto.
  apply L.eq_refl.
Qed.

Definition ge (x y: t) : Prop :=
   p, L.ge (get p x) (get p y).

Lemma ge_refl: x y, eq x y ge x y.
Proof.
  unfold ge, eq; intros. apply L.ge_refl. auto.
Qed.

Lemma ge_trans: x y z, ge x y ge y z ge x z.
Proof.
  unfold ge; intros. apply L.ge_trans with (get p y); auto.
Qed.

Definition bot : t := PTree.empty _.

Lemma get_bot: p, get p bot = L.bot.
Proof.
  unfold bot, get; intros; simpl. rewrite PTree.gempty. auto.
Qed.

Lemma ge_bot: x, ge x bot.
Proof.
  unfold ge; intros. rewrite get_bot. apply L.ge_bot.
Qed.

A combine operation over the type PTree.t L.t that attempts to share its result with its arguments.

Section COMBINE.

Variable f: option L.t option L.t option L.t.
Hypothesis f_none_none: f None None = None.

Definition opt_eq (ox oy: option L.t) : Prop :=
  match ox, oy with
  | None, NoneTrue
  | Some x, Some yL.eq x y
  | _, _False
  end.

Lemma opt_eq_refl: ox, opt_eq ox ox.
Proof.
  intros. unfold opt_eq. destruct ox. apply L.eq_refl. auto.
Qed.

Lemma opt_eq_sym: ox oy, opt_eq ox oy opt_eq oy ox.
Proof.
  unfold opt_eq. destruct ox; destruct oy; auto. apply L.eq_sym.
Qed.

Lemma opt_eq_trans: ox oy oz, opt_eq ox oy opt_eq oy oz opt_eq ox oz.
Proof.
  unfold opt_eq. destruct ox; destruct oy; destruct oz; intuition.
  eapply L.eq_trans; eauto.
Qed.

Definition opt_beq (ox oy: option L.t) : bool :=
  match ox, oy with
  | None, Nonetrue
  | Some x, Some yL.beq x y
  | _, _false
  end.

Lemma opt_beq_correct:
   ox oy, opt_beq ox oy = true opt_eq ox oy.
Proof.
  unfold opt_beq, opt_eq. destruct ox; destruct oy; try congruence.
  intros. apply L.beq_correct; auto.
  auto.
Qed.

Definition tree_eq (m1 m2: PTree.t L.t) : Prop :=
   i, opt_eq (PTree.get i m1) (PTree.get i m2).

Lemma tree_eq_refl: m, tree_eq m m.
Proof. intros; red; intros; apply opt_eq_refl. Qed.

Lemma tree_eq_sym: m1 m2, tree_eq m1 m2 tree_eq m2 m1.
Proof. intros; red; intros; apply opt_eq_sym; auto. Qed.

Lemma tree_eq_trans: m1 m2 m3, tree_eq m1 m2 tree_eq m2 m3 tree_eq m1 m3.
Proof. intros; red; intros; apply opt_eq_trans with (PTree.get i m2); auto. Qed.

Lemma tree_eq_node:
   l1 o1 r1 l2 o2 r2,
  tree_eq l1 l2 tree_eq r1 r2 opt_eq o1 o2
  tree_eq (PTree.Node l1 o1 r1) (PTree.Node l2 o2 r2).
Proof.
  intros; red; intros. destruct i; simpl; auto.
Qed.

Lemma tree_eq_node':
   l1 o1 r1 l2 o2 r2,
  tree_eq l1 l2 tree_eq r1 r2 opt_eq o1 o2
  tree_eq (PTree.Node l1 o1 r1) (PTree.Node' l2 o2 r2).
Proof.
  intros; red; intros. rewrite PTree.gnode'. apply tree_eq_node; auto.
Qed.

Lemma tree_eq_node'':
   l1 o1 r1 l2 o2 r2,
  tree_eq l1 l2 tree_eq r1 r2 opt_eq o1 o2
  tree_eq (PTree.Node' l1 o1 r1) (PTree.Node' l2 o2 r2).
Proof.
  intros; red; intros. repeat rewrite PTree.gnode'. apply tree_eq_node; auto.
Qed.

Hint Resolve opt_beq_correct opt_eq_refl opt_eq_sym
             tree_eq_refl tree_eq_sym
             tree_eq_node tree_eq_node' tree_eq_node'' : combine.

Inductive changed: Type := Unchanged | Changed (m: PTree.t L.t).

Fixpoint combine_l (m : PTree.t L.t) {struct m} : changed :=
  match m with
  | PTree.Leaf
      Unchanged
  | PTree.Node l o r
      let o' := f o None in
      match combine_l l, combine_l r with
      | Unchanged, Unchangedif opt_beq o' o then Unchanged else Changed (PTree.Node' l o' r)
      | Unchanged, Changed r'Changed (PTree.Node' l o' r')
      | Changed l', UnchangedChanged (PTree.Node' l' o' r)
      | Changed l', Changed r'Changed (PTree.Node' l' o' r')
      end
  end.

Lemma combine_l_eq:
   m,
  tree_eq (match combine_l m with Unchangedm | Changed m'm' end)
          (PTree.xcombine_l f m).
Proof.
  induction m; simpl.
  auto with combine.
  destruct (combine_l m1) as [ | l']; destruct (combine_l m2) as [ | r'];
  auto with combine.
  case_eq (opt_beq (f o None) o); auto with combine.
Qed.

Fixpoint combine_r (m : PTree.t L.t) {struct m} : changed :=
  match m with
  | PTree.Leaf
      Unchanged
  | PTree.Node l o r
      let o' := f None o in
      match combine_r l, combine_r r with
      | Unchanged, Unchangedif opt_beq o' o then Unchanged else Changed (PTree.Node' l o' r)
      | Unchanged, Changed r'Changed (PTree.Node' l o' r')
      | Changed l', UnchangedChanged (PTree.Node' l' o' r)
      | Changed l', Changed r'Changed (PTree.Node' l' o' r')
      end
  end.

Lemma combine_r_eq:
   m,
  tree_eq (match combine_r m with Unchangedm | Changed m'm' end)
          (PTree.xcombine_r f m).
Proof.
  induction m; simpl.
  auto with combine.
  destruct (combine_r m1) as [ | l']; destruct (combine_r m2) as [ | r'];
  auto with combine.
  case_eq (opt_beq (f None o) o); auto with combine.
Qed.

Inductive changed2 : Type :=
  | Same
  | Same1
  | Same2
  | CC(m: PTree.t L.t).

Fixpoint xcombine (m1 m2 : PTree.t L.t) {struct m1} : changed2 :=
    match m1, m2 with
    | PTree.Leaf, PTree.Leaf
        Same
    | PTree.Leaf, _
        match combine_r m2 with
        | UnchangedSame2
        | Changed mCC m
        end
    | _, PTree.Leaf
        match combine_l m1 with
        | UnchangedSame1
        | Changed mCC m
        end
    | PTree.Node l1 o1 r1, PTree.Node l2 o2 r2
        let o := f o1 o2 in
        match xcombine l1 l2, xcombine r1 r2 with
        | Same, Same
            match opt_beq o o1, opt_beq o o2 with
            | true, trueSame
            | true, falseSame1
            | false, trueSame2
            | false, falseCC(PTree.Node' l1 o r1)
            end
        | Same1, Same | Same, Same1 | Same1, Same1
            if opt_beq o o1 then Same1 else CC(PTree.Node' l1 o r1)
        | Same2, Same | Same, Same2 | Same2, Same2
            if opt_beq o o2 then Same2 else CC(PTree.Node' l2 o r2)
        | Same1, Same2CC(PTree.Node' l1 o r2)
        | (Same|Same1), CC rCC(PTree.Node' l1 o r)
        | Same2, Same1CC(PTree.Node' l2 o r1)
        | Same2, CC rCC(PTree.Node' l2 o r)
        | CC l, (Same|Same1) ⇒ CC(PTree.Node' l o r1)
        | CC l, Same2CC(PTree.Node' l o r2)
        | CC l, CC rCC(PTree.Node' l o r)
        end
    end.

Lemma xcombine_eq:
   m1 m2,
  match xcombine m1 m2 with
  | Sametree_eq m1 (PTree.combine f m1 m2) tree_eq m2 (PTree.combine f m1 m2)
  | Same1tree_eq m1 (PTree.combine f m1 m2)
  | Same2tree_eq m2 (PTree.combine f m1 m2)
  | CC mtree_eq m (PTree.combine f m1 m2)
  end.
Proof.
Opaque combine_l combine_r PTree.xcombine_l PTree.xcombine_r.
  induction m1; destruct m2; simpl.
  split; apply tree_eq_refl.
  generalize (combine_r_eq (PTree.Node m2_1 o m2_2)).
  destruct (combine_r (PTree.Node m2_1 o m2_2)); auto.
  generalize (combine_l_eq (PTree.Node m1_1 o m1_2)).
  destruct (combine_l (PTree.Node m1_1 o m1_2)); auto.
  generalize (IHm1_1 m2_1) (IHm1_2 m2_2).
  destruct (xcombine m1_1 m2_1);
  destruct (xcombine m1_2 m2_2); auto with combine;
  intuition; case_eq (opt_beq (f o o0) o); case_eq (opt_beq (f o o0) o0); auto with combine.
Qed.

Definition combine (m1 m2: PTree.t L.t) : PTree.t L.t :=
  match xcombine m1 m2 with
  | Same|Same1m1
  | Same2m2
  | CC mm
  end.

Lemma gcombine:
   m1 m2 i, opt_eq (PTree.get i (combine m1 m2)) (f (PTree.get i m1) (PTree.get i m2)).
Proof.
  intros.
  assert (tree_eq (combine m1 m2) (PTree.combine f m1 m2)).
  unfold combine.
  generalize (xcombine_eq m1 m2).
  destruct (xcombine m1 m2); tauto.
  eapply opt_eq_trans. apply H. rewrite PTree.gcombine; auto. apply opt_eq_refl.
Qed.

End COMBINE.

Definition lub (x y: t) : t :=
  combine
    (fun a b
       match a, b with
       | Some u, Some vSome (L.lub u v)
       | None, _b
       | _, Nonea
       end)
    x y.

Lemma gcombine_bot:
   f t1 t2 p,
  f None None = None
  L.eq (get p (combine f t1 t2))
       (match f t1!p t2!p with Some xx | NoneL.bot end).
Proof.
  intros. unfold get. generalize (gcombine f H t1 t2 p). unfold opt_eq.
  destruct ((combine f t1 t2)!p); destruct (f t1!p t2!p).
  auto. contradiction. contradiction. intros; apply L.eq_refl.
Qed.

Lemma ge_lub_left:
   x y, ge (lub x y) x.
Proof.
  unfold ge, lub; intros.
  eapply L.ge_trans. apply L.ge_refl. apply gcombine_bot; auto.
  unfold get. destruct x!p. destruct y!p.
  apply L.ge_lub_left.
  apply L.ge_refl. apply L.eq_refl.
  apply L.ge_bot.
Qed.

Lemma ge_lub_right:
   x y, ge (lub x y) y.
Proof.
  unfold ge, lub; intros.
  eapply L.ge_trans. apply L.ge_refl. apply gcombine_bot; auto.
  unfold get. destruct y!p. destruct x!p.
  apply L.ge_lub_right.
  apply L.ge_refl. apply L.eq_refl.
  apply L.ge_bot.
Qed.

End LPMap1.

Given a semi-lattice with top L, the following functor implements a semi-lattice-with-top structure over finite maps from positive numbers to L.t. The default value for these maps is L.top. Bottom elements are smashed.

Module LPMap(L: SEMILATTICE_WITH_TOP) <: SEMILATTICE_WITH_TOP.

Inductive t' : Type :=
  | Bot: t'
  | Top_except: PTree.t L.t t'.

Definition t: Type := t'.

Definition get (p: positive) (x: t) : L.t :=
  match x with
  | BotL.bot
  | Top_except mmatch m!p with NoneL.top | Some xx end
  end.

Definition set (p: positive) (v: L.t) (x: t) : t :=
  match x with
  | BotBot
  | Top_except m
      if L.beq v L.bot
      then Bot
      else Top_except (if L.beq v L.top then PTree.remove p m else PTree.set p v m)
  end.

Lemma gsspec:
   p v x q,
  x Bot ¬L.eq v L.bot
  L.eq (get q (set p v x)) (if peq q p then v else get q x).
Proof.
  intros. unfold set. destruct x. congruence.
  destruct (L.beq v L.bot) eqn:EBOT.
  elim H0. apply L.beq_correct; auto.
  destruct (L.beq v L.top) eqn:ETOP; simpl.
  rewrite PTree.grspec. unfold PTree.elt_eq. destruct (peq q p).
  apply L.eq_sym. apply L.beq_correct; auto.
  apply L.eq_refl.
  rewrite PTree.gsspec. destruct (peq q p); apply L.eq_refl.
Qed.

Definition eq (x y: t) : Prop :=
   p, L.eq (get p x) (get p y).

Lemma eq_refl: x, eq x x.
Proof.
  unfold eq; intros. apply L.eq_refl.
Qed.

Lemma eq_sym: x y, eq x y eq y x.
Proof.
  unfold eq; intros. apply L.eq_sym; auto.
Qed.

Lemma eq_trans: x y z, eq x y eq y z eq x z.
Proof.
  unfold eq; intros. eapply L.eq_trans; eauto.
Qed.

Definition beq (x y: t) : bool :=
  match x, y with
  | Bot, Bottrue
  | Top_except m, Top_except nPTree.beq L.beq m n
  | _, _false
  end.

Lemma beq_correct: x y, beq x y = true eq x y.
Proof.
  destruct x; destruct y; simpl; intro; try congruence.
  apply eq_refl.
  red; intro; simpl.
  rewrite PTree.beq_correct in H. generalize (H p).
  destruct (t0!p); destruct (t1!p); intuition.
  apply L.beq_correct; auto.
  apply L.eq_refl.
Qed.

Definition ge (x y: t) : Prop :=
   p, L.ge (get p x) (get p y).

Lemma ge_refl: x y, eq x y ge x y.
Proof.
  unfold ge, eq; intros. apply L.ge_refl. auto.
Qed.

Lemma ge_trans: x y z, ge x y ge y z ge x z.
Proof.
  unfold ge; intros. apply L.ge_trans with (get p y); auto.
Qed.

Definition bot := Bot.

Lemma get_bot: p, get p bot = L.bot.
Proof.
  unfold bot; intros; simpl. auto.
Qed.

Lemma ge_bot: x, ge x bot.
Proof.
  unfold ge; intros. rewrite get_bot. apply L.ge_bot.
Qed.

Definition top := Top_except (PTree.empty L.t).

Lemma get_top: p, get p top = L.top.
Proof.
  unfold top; intros; simpl. rewrite PTree.gempty. auto.
Qed.

Lemma ge_top: x, ge top x.
Proof.
  unfold ge; intros. rewrite get_top. apply L.ge_top.
Qed.

Module LM := LPMap1(L).

Definition opt_lub (x y: L.t) : option L.t :=
  let z := L.lub x y in
  if L.beq z L.top then None else Some z.

Definition lub (x y: t) : t :=
  match x, y with
  | Bot, _y
  | _, Botx
  | Top_except m, Top_except n
      Top_except
        (LM.combine
           (fun a b
              match a, b with
              | Some u, Some vopt_lub u v
              | _, _None
              end)
           m n)
  end.

Lemma gcombine_top:
   f t1 t2 p,
  f None None = None
  L.eq (get p (Top_except (LM.combine f t1 t2)))
       (match f t1!p t2!p with Some xx | NoneL.top end).
Proof.
  intros. simpl. generalize (LM.gcombine f H t1 t2 p). unfold LM.opt_eq.
  destruct ((LM.combine f t1 t2)!p); destruct (f t1!p t2!p).
  auto. contradiction. contradiction. intros; apply L.eq_refl.
Qed.

Lemma ge_lub_left:
   x y, ge (lub x y) x.
Proof.
  unfold ge, lub; intros. destruct x; destruct y.
  rewrite get_bot. apply L.ge_bot.
  rewrite get_bot. apply L.ge_bot.
  apply L.ge_refl. apply L.eq_refl.
  eapply L.ge_trans. apply L.ge_refl. apply gcombine_top; auto.
  unfold get. destruct t0!p. destruct t1!p.
  unfold opt_lub. destruct (L.beq (L.lub t2 t3) L.top) eqn:E.
  apply L.ge_top. apply L.ge_lub_left.
  apply L.ge_top.
  apply L.ge_top.
Qed.

Lemma ge_lub_right:
   x y, ge (lub x y) y.
Proof.
  unfold ge, lub; intros. destruct x; destruct y.
  rewrite get_bot. apply L.ge_bot.
  apply L.ge_refl. apply L.eq_refl.
  rewrite get_bot. apply L.ge_bot.
  eapply L.ge_trans. apply L.ge_refl. apply gcombine_top; auto.
  unfold get. destruct t0!p; destruct t1!p.
  unfold opt_lub. destruct (L.beq (L.lub t2 t3) L.top) eqn:E.
  apply L.ge_top. apply L.ge_lub_right.
  apply L.ge_top.
  apply L.ge_top.
  apply L.ge_top.
Qed.

End LPMap.

Semi-lattice over a set.

Given a set S: FSetInterface.S, the following functor implements a semi-lattice over these sets, ordered by inclusion.

Module LFSet (S: FSetInterface.WS) <: SEMILATTICE.

  Definition t := S.t.

  Definition eq (x y: t) := S.Equal x y.
  Definition eq_refl: x, eq x x := S.eq_refl.
  Definition eq_sym: x y, eq x y eq y x := S.eq_sym.
  Definition eq_trans: x y z, eq x y eq y z eq x z := S.eq_trans.
  Definition beq: t t bool := S.equal.
  Definition beq_correct: x y, beq x y = true eq x y := S.equal_2.

  Definition ge (x y: t) := S.Subset y x.
  Lemma ge_refl: x y, eq x y ge x y.
  Proof.
    unfold eq, ge, S.Equal, S.Subset; intros. firstorder.
  Qed.
  Lemma ge_trans: x y z, ge x y ge y z ge x z.
  Proof.
    unfold ge, S.Subset; intros. eauto.
  Qed.

  Definition bot: t := S.empty.
  Lemma ge_bot: x, ge x bot.
  Proof.
    unfold ge, bot, S.Subset; intros. elim (S.empty_1 H).
  Qed.

  Definition lub: t t t := S.union.

  Lemma ge_lub_left: x y, ge (lub x y) x.
  Proof.
    unfold lub, ge, S.Subset; intros. apply S.union_2; auto.
  Qed.

  Lemma ge_lub_right: x y, ge (lub x y) y.
  Proof.
    unfold lub, ge, S.Subset; intros. apply S.union_3; auto.
  Qed.

End LFSet.

Flat semi-lattice

Given a type with decidable equality X, the following functor returns a semi-lattice structure over X.t complemented with a top and a bottom element. The ordering is the flat ordering Bot < Inj x < Top.

Module LFlat(X: EQUALITY_TYPE) <: SEMILATTICE_WITH_TOP.

Inductive t' : Type :=
  | Bot: t'
  | Inj: X.t t'
  | Top: t'.

Definition t : Type := t'.

Definition eq (x y: t) := (x = y).
Definition eq_refl: x, eq x x := (@eq_refl t).
Definition eq_sym: x y, eq x y eq y x := (@eq_sym t).
Definition eq_trans: x y z, eq x y eq y z eq x z := (@eq_trans t).

Definition beq (x y: t) : bool :=
  match x, y with
  | Bot, Bottrue
  | Inj u, Inj vif X.eq u v then true else false
  | Top, Toptrue
  | _, _false
  end.

Lemma beq_correct: x y, beq x y = true eq x y.
Proof.
  unfold eq. destruct x; destruct y; simpl; try congruence; intro.
  destruct (X.eq t0 t1); congruence.
Qed.

Definition ge (x y: t) : Prop :=
  match x, y with
  | Top, _True
  | _, BotTrue
  | Inj a, Inj ba = b
  | _, _False
  end.

Lemma ge_refl: x y, eq x y ge x y.
Proof.
  unfold eq, ge; intros; subst y; destruct x; auto.
Qed.

Lemma ge_trans: x y z, ge x y ge y z ge x z.
Proof.
  unfold ge; destruct x; destruct y; try destruct z; intuition.
  transitivity t1; auto.
Qed.

Definition bot: t := Bot.

Lemma ge_bot: x, ge x bot.
Proof.
  destruct x; simpl; auto.
Qed.

Definition top: t := Top.

Lemma ge_top: x, ge top x.
Proof.
  destruct x; simpl; auto.
Qed.

Definition lub (x y: t) : t :=
  match x, y with
  | Bot, _y
  | _, Botx
  | Top, _Top
  | _, TopTop
  | Inj a, Inj bif X.eq a b then Inj a else Top
  end.

Lemma ge_lub_left: x y, ge (lub x y) x.
Proof.
  destruct x; destruct y; simpl; auto.
  case (X.eq t0 t1); simpl; auto.
Qed.

Lemma ge_lub_right: x y, ge (lub x y) y.
Proof.
  destruct x; destruct y; simpl; auto.
  case (X.eq t0 t1); simpl; auto.
Qed.

End LFlat.

Boolean semi-lattice

This semi-lattice has only two elements, bot and top, trivially ordered.

Module LBoolean <: SEMILATTICE_WITH_TOP.

Definition t := bool.

Definition eq (x y: t) := (x = y).
Definition eq_refl: x, eq x x := (@eq_refl t).
Definition eq_sym: x y, eq x y eq y x := (@eq_sym t).
Definition eq_trans: x y z, eq x y eq y z eq x z := (@eq_trans t).

Definition beq : t t bool := eqb.

Lemma beq_correct: x y, beq x y = true eq x y.
Proof eqb_prop.

Definition ge (x y: t) : Prop := x = y x = true.

Lemma ge_refl: x y, eq x y ge x y.
Proof. unfold ge; tauto. Qed.

Lemma ge_trans: x y z, ge x y ge y z ge x z.
Proof. unfold ge; intuition congruence. Qed.

Definition bot := false.

Lemma ge_bot: x, ge x bot.
Proof. destruct x; compute; tauto. Qed.

Definition top := true.

Lemma ge_top: x, ge top x.
Proof. unfold ge, top; tauto. Qed.

Definition lub (x y: t) := x || y.

Lemma ge_lub_left: x y, ge (lub x y) x.
Proof. destruct x; destruct y; compute; tauto. Qed.

Lemma ge_lub_right: x y, ge (lub x y) y.
Proof. destruct x; destruct y; compute; tauto. Qed.

End LBoolean.

Option semi-lattice

This lattice adds a top element (represented by None) to a given semi-lattice (whose elements are injected via Some).

Module LOption(L: SEMILATTICE) <: SEMILATTICE_WITH_TOP.

Definition t: Type := option L.t.

Definition eq (x y: t) : Prop :=
  match x, y with
  | None, NoneTrue
  | Some x1, Some y1L.eq x1 y1
  | _, _False
  end.

Lemma eq_refl: x, eq x x.
Proof.
  unfold eq; intros; destruct x. apply L.eq_refl. auto.
Qed.

Lemma eq_sym: x y, eq x y eq y x.
Proof.
  unfold eq; intros; destruct x; destruct y; auto. apply L.eq_sym; auto.
Qed.

Lemma eq_trans: x y z, eq x y eq y z eq x z.
Proof.
  unfold eq; intros; destruct x; destruct y; destruct z; auto.
  eapply L.eq_trans; eauto.
  contradiction.
Qed.

Definition beq (x y: t) : bool :=
  match x, y with
  | None, Nonetrue
  | Some x1, Some y1L.beq x1 y1
  | _, _false
  end.

Lemma beq_correct: x y, beq x y = true eq x y.
Proof.
  unfold beq, eq; intros; destruct x; destruct y.
  apply L.beq_correct; auto.
  discriminate. discriminate. auto.
Qed.

Definition ge (x y: t) : Prop :=
  match x, y with
  | None, _True
  | _, NoneFalse
  | Some x1, Some y1L.ge x1 y1
  end.

Lemma ge_refl: x y, eq x y ge x y.
Proof.
  unfold eq, ge; intros; destruct x; destruct y.
  apply L.ge_refl; auto.
  auto. elim H. auto.
Qed.

Lemma ge_trans: x y z, ge x y ge y z ge x z.
Proof.
  unfold ge; intros; destruct x; destruct y; destruct z; auto.
  eapply L.ge_trans; eauto. contradiction.
Qed.

Definition bot : t := Some L.bot.

Lemma ge_bot: x, ge x bot.
Proof.
  unfold ge, bot; intros. destruct x; auto. apply L.ge_bot.
Qed.

Definition lub (x y: t) : t :=
  match x, y with
  | None, _None
  | _, NoneNone
  | Some x1, Some y1Some (L.lub x1 y1)
  end.

Lemma ge_lub_left: x y, ge (lub x y) x.
Proof.
  unfold ge, lub; intros; destruct x; destruct y; auto. apply L.ge_lub_left.
Qed.

Lemma ge_lub_right: x y, ge (lub x y) y.
Proof.
  unfold ge, lub; intros; destruct x; destruct y; auto. apply L.ge_lub_right.
Qed.

Definition top : t := None.

Lemma ge_top: x, ge top x.
Proof.
  unfold ge, top; intros. auto.
Qed.

End LOption.