Library UniMath.OrderTheory.Lattice.Examples.Subsets
Require Import UniMath.Foundations.Preamble.
Require Import UniMath.Foundations.PartA.
Require Import UniMath.Foundations.Sets.
Require Import UniMath.MoreFoundations.Sets.
Require Export UniMath.MoreFoundations.Propositions.
Require Export UniMath.MoreFoundations.Subtypes.
Require Import UniMath.Algebra.BinaryOperations.
Require Import UniMath.OrderTheory.Lattice.Lattice.
Require Import UniMath.OrderTheory.Lattice.Bounded.
Require Import UniMath.OrderTheory.Lattice.Distributive.
Require Import UniMath.OrderTheory.Lattice.Complement.
Require Import UniMath.OrderTheory.Lattice.Boolean.
Section Subsets.
Context {X : hSet}.
Definition intersection_binop : binop (subtype_set X).
Show proof.
Lemma isassoc_intersection_binop : isassoc intersection_binop.
Show proof.
    intros W Y Z.
apply (invweq (hsubtype_univalence _ _)), subtype_equal_cond.
use make_dirprod; cbn; intros z f b; induction b; cbn in *.
+
apply (invweq (hsubtype_univalence _ _)), subtype_equal_cond.
use make_dirprod; cbn; intros z f b; induction b; cbn in *.
+
        exact (f false).
+ intro b; induction b; cbn in *.
* exact (f true).
* exact (f false true).
+ exact (f false false).
+ intro b; induction b; cbn in *.
* exact (f true).
* exact (f false true).
+ exact (f false false).
Lemma iscomm_intersection_binop : iscomm intersection_binop.
Show proof.
    intros ? ?; unfold intersection_binop, infinitary_op_to_binop; cbn.
apply (invweq (hsubtype_univalence _ _)), subtype_equal_cond.
use make_dirprod; intro; cbn; intros f b; induction b.
- exact (f false).
- exact (f true).
- exact (f false).
- exact (f true).
apply (invweq (hsubtype_univalence _ _)), subtype_equal_cond.
use make_dirprod; intro; cbn; intros f b; induction b.
- exact (f false).
- exact (f true).
- exact (f false).
- exact (f true).
Definition union_binop : binop (subtype_set X).
Show proof.
Local Lemma squash_to_prop_ishinh {Y Q : UU} :
∥ Y ∥ → (Y → ∥ Q ∥) → ∥ Q ∥.
Show proof.
Lemma isassoc_union_binop : isassoc union_binop.
Show proof.
    intros ? ? ?.
apply (invweq (hsubtype_univalence _ _)), subtype_equal_cond.
use make_dirprod; cbn; intros ? ain;
apply (squash_to_prop_ishinh ain);
clear ain; intro ain; induction ain as [b bin].
- induction b; cbn in bin.
+ apply (squash_to_prop_ishinh bin); clear bin; intro bin.
induction bin as [c cin].
induction c.
* apply hinhpr; exists true; assumption.
* apply hinhpr; exists false; cbn in *.
apply hinhpr; exists true; assumption.
+ do 2 (apply hinhpr; exists false); assumption.
- induction b; cbn in bin.
+ do 2 (apply hinhpr; exists true); assumption.
+ apply (squash_to_prop_ishinh bin); clear bin; intro bin.
induction bin as [c cin].
induction c.
* apply hinhpr; exists true; cbn in *.
apply hinhpr; exists false; assumption.
* apply hinhpr; exists false; assumption.
apply (invweq (hsubtype_univalence _ _)), subtype_equal_cond.
use make_dirprod; cbn; intros ? ain;
apply (squash_to_prop_ishinh ain);
clear ain; intro ain; induction ain as [b bin].
- induction b; cbn in bin.
+ apply (squash_to_prop_ishinh bin); clear bin; intro bin.
induction bin as [c cin].
induction c.
* apply hinhpr; exists true; assumption.
* apply hinhpr; exists false; cbn in *.
apply hinhpr; exists true; assumption.
+ do 2 (apply hinhpr; exists false); assumption.
- induction b; cbn in bin.
+ do 2 (apply hinhpr; exists true); assumption.
+ apply (squash_to_prop_ishinh bin); clear bin; intro bin.
induction bin as [c cin].
induction c.
* apply hinhpr; exists true; cbn in *.
apply hinhpr; exists false; assumption.
* apply hinhpr; exists false; assumption.
Lemma iscomm_union_binop : iscomm union_binop.
intros ? ?; unfold union_binop, infinitary_op_to_binop; cbn.
apply (invweq (hsubtype_univalence _ _)), subtype_equal_cond.
use make_dirprod; intro; cbn; intros ain;
apply (squash_to_prop_ishinh ain); clear ain; intro ain;
induction ain as [b bin]; induction b; cbn in *;
apply hinhpr.
- exists false; assumption.
- exists true; assumption.
- exists false; assumption.
- exists true; assumption.
Qed.
Lemma subset_lattice : lattice (subtype_set X).
Show proof.
    - exact union_binop. 
    - 
TODO: constructor for this 
      apply make_dirprod; [apply make_dirprod|apply make_dirprod; [apply make_dirprod|apply make_dirprod]].
+ apply isassoc_intersection_binop.
+ apply iscomm_intersection_binop.
+ apply isassoc_union_binop.
+ apply iscomm_union_binop.
+ intros ? ?.
apply (invweq (hsubtype_univalence _ _)), subtype_equal_cond.
use make_dirprod.
* intros ? f; exact (f true).
* intros ? ?.
intros b; induction b; cbn.
-- assumption.
-- apply hinhpr; exists true; assumption.
+ intros ? ?.
apply (invweq (hsubtype_univalence _ _)), subtype_equal_cond.
use make_dirprod.
* intros ? f; cbn in f.
refine (hinhuniv _ f); clear f; intro f.
induction f as [b bin]; induction b; cbn in bin.
-- assumption.
-- apply (bin true).
* intros ? ?; apply hinhpr; exists true; assumption.
+ apply isassoc_intersection_binop.
+ apply iscomm_intersection_binop.
+ apply isassoc_union_binop.
+ apply iscomm_union_binop.
+ intros ? ?.
apply (invweq (hsubtype_univalence _ _)), subtype_equal_cond.
use make_dirprod.
* intros ? f; exact (f true).
* intros ? ?.
intros b; induction b; cbn.
-- assumption.
-- apply hinhpr; exists true; assumption.
+ intros ? ?.
apply (invweq (hsubtype_univalence _ _)), subtype_equal_cond.
use make_dirprod.
* intros ? f; cbn in f.
refine (hinhuniv _ f); clear f; intro f.
induction f as [b bin]; induction b; cbn in bin.
-- assumption.
-- apply (bin true).
* intros ? ?; apply hinhpr; exists true; assumption.
Lemma subset_lattice_is_bounded :
bounded_latticeop subset_lattice (emptysubtype X) (totalsubtype X).
Show proof.
TODO: constructor 
    use make_dirprod.
- intros x; cbn.
apply (invweq (hsubtype_univalence _ _)), subtype_equal_cond;
use make_dirprod.
+ intros ? in_union.
refine (hinhuniv _ in_union); clear in_union; intro in_union.
induction in_union as [b bin]; induction b; cbn in bin.
* induction bin. * assumption.
+ intros ? ?; apply hinhpr; exists false; assumption.
- intros x; cbn.
apply (invweq (hsubtype_univalence _ _)), subtype_equal_cond;
use make_dirprod.
+ intros ? in_intersection; exact (in_intersection false).
+ intros ? ? b; induction b; cbn.
* exact tt. * assumption.
- intros x; cbn.
apply (invweq (hsubtype_univalence _ _)), subtype_equal_cond;
use make_dirprod.
+ intros ? in_union.
refine (hinhuniv _ in_union); clear in_union; intro in_union.
induction in_union as [b bin]; induction b; cbn in bin.
* induction bin. * assumption.
+ intros ? ?; apply hinhpr; exists false; assumption.
- intros x; cbn.
apply (invweq (hsubtype_univalence _ _)), subtype_equal_cond;
use make_dirprod.
+ intros ? in_intersection; exact (in_intersection false).
+ intros ? ? b; induction b; cbn.
* exact tt. * assumption.
Using LEM, we can show the lattice is complemented 
  Lemma subset_lattice_is_complemented :
LEM -> complemented_structure (make_bounded_lattice subset_lattice_is_bounded).
Show proof.
Definition subset_bounded_lattice : bounded_lattice (subtype_set X).
Show proof.
Lemma subset_lattice_is_distributive : is_distributive subset_lattice.
Show proof.
LEM -> complemented_structure (make_bounded_lattice subset_lattice_is_bounded).
Show proof.
    intros lem sub.
exists (subtype_complement sub).
use make_dirprod.
- apply (invweq (hsubtype_univalence _ _)).
eapply (subtype_complement_union lem).
+ exists true; reflexivity.
+ exists false; reflexivity.
-
exists (subtype_complement sub).
use make_dirprod.
- apply (invweq (hsubtype_univalence _ _)).
eapply (subtype_complement_union lem).
+ exists true; reflexivity.
+ exists false; reflexivity.
-
We don't need LEM for this branch. 
      apply (invweq (hsubtype_univalence _ _)).
eapply subtype_complement_intersection_empty.
+ exists true; reflexivity.
+ exists false; reflexivity.
eapply subtype_complement_intersection_empty.
+ exists true; reflexivity.
+ exists false; reflexivity.
Definition subset_bounded_lattice : bounded_lattice (subtype_set X).
Show proof.
    use make_bounded_lattice.
- exact subset_lattice.
- exact (emptysubtype X).
- exact (totalsubtype X).
- exact subset_lattice_is_bounded.
- exact subset_lattice.
- exact (emptysubtype X).
- exact (totalsubtype X).
- exact subset_lattice_is_bounded.
Lemma subset_lattice_is_distributive : is_distributive subset_lattice.
Show proof.
  Abort.
Definition subset_lattice_is_boolean :
LEM -> is_boolean subset_bounded_lattice.
Proof.
intros lem.
use make_is_boolean.
2: apply (subset_lattice_is_complemented lem).
Abort.
End Subsets.
Definition subset_lattice_is_boolean :
LEM -> is_boolean subset_bounded_lattice.
Proof.
intros lem.
use make_is_boolean.
2: apply (subset_lattice_is_complemented lem).
Abort.
End Subsets.