Library UniMath.Bicategories.DoubleCategories.Examples.HorizontalDual
Require Import UniMath.MoreFoundations.All.
Require Import UniMath.CategoryTheory.Core.Prelude.
Require Import UniMath.CategoryTheory.TwoSidedDisplayedCats.TwoSidedDispCat.
Require Import UniMath.Bicategories.Core.Bicat.
Import Bicat.Notations.
Require Import UniMath.Bicategories.Core.Invertible_2cells.
Require Import UniMath.Bicategories.Core.Univalence.
Require Import UniMath.Bicategories.Core.UnivalenceOp.
Require Import UniMath.Bicategories.Core.Examples.OpMorBicat.
Require Import UniMath.Bicategories.Core.Examples.OpCellBicat.
Require Import UniMath.Bicategories.DoubleCategories.DoubleBicat.VerityDoubleBicat.
Require Import UniMath.Bicategories.DoubleCategories.DoubleBicat.DerivedLaws.
Require Import UniMath.Bicategories.DoubleCategories.DoubleBicat.CellsAndSquares.
Require Import UniMath.Bicategories.DoubleCategories.DoubleBicat.UnderlyingCats.
Require Import UniMath.Bicategories.DoubleCategories.DoubleBicat.LocalUnivalence.
Local Open Scope cat.
Local Open Scope double_bicat.
Section HorizontalDual.
Context (B : verity_double_bicat).
Let π : bicat := ver_bicat_of_verity_double_bicat B.
Require Import UniMath.CategoryTheory.Core.Prelude.
Require Import UniMath.CategoryTheory.TwoSidedDisplayedCats.TwoSidedDispCat.
Require Import UniMath.Bicategories.Core.Bicat.
Import Bicat.Notations.
Require Import UniMath.Bicategories.Core.Invertible_2cells.
Require Import UniMath.Bicategories.Core.Univalence.
Require Import UniMath.Bicategories.Core.UnivalenceOp.
Require Import UniMath.Bicategories.Core.Examples.OpMorBicat.
Require Import UniMath.Bicategories.Core.Examples.OpCellBicat.
Require Import UniMath.Bicategories.DoubleCategories.DoubleBicat.VerityDoubleBicat.
Require Import UniMath.Bicategories.DoubleCategories.DoubleBicat.DerivedLaws.
Require Import UniMath.Bicategories.DoubleCategories.DoubleBicat.CellsAndSquares.
Require Import UniMath.Bicategories.DoubleCategories.DoubleBicat.UnderlyingCats.
Require Import UniMath.Bicategories.DoubleCategories.DoubleBicat.LocalUnivalence.
Local Open Scope cat.
Local Open Scope double_bicat.
Section HorizontalDual.
Context (B : verity_double_bicat).
Let π : bicat := ver_bicat_of_verity_double_bicat B.
Definition horizontal_dual_hor_bicat
: bicat
:= op1_bicat (hor_bicat_of_verity_double_bicat B).
Definition horizontal_dual_twosided_disp_cat_data
: twosided_disp_cat_data horizontal_dual_hor_bicat horizontal_dual_hor_bicat.
Proof.
simple refine ((_ ,, _) ,, (_ ,, _)).
- exact (Ξ» (x y : B), x -|-> y).
- exact (Ξ» (xβ xβ yβ yβ : B)
(vβ : xβ -|-> yβ) (vβ : xβ -|-> yβ)
(hβ : xβ --> xβ) (hβ : yβ --> yβ),
square_double_bicat hβ hβ vβ vβ).
- exact (Ξ» (x y : B) (v : x -|-> y), id_h_square_bicat _).
- exact (Ξ» (xβ xβ xβ yβ yβ yβ : B)
(vβ : xβ -|-> yβ) (vβ : xβ -|-> yβ) (vβ : xβ -|-> yβ)
(hβ : xβ --> xβ) (hβ : xβ --> xβ)
(kβ : yβ --> yβ) (kβ : yβ --> yβ)
(sβ : square_double_bicat hβ kβ vβ vβ)
(sβ : square_double_bicat hβ kβ vβ vβ),
sβ βh sβ).
Defined.
Definition horizontal_dual_ver_sq_bicat
: ver_sq_bicat.
Proof.
use make_ver_sq_bicat.
- exact horizontal_dual_hor_bicat.
- exact horizontal_dual_twosided_disp_cat_data.
Defined.
Definition horizontal_dual_ver_sq_bicat_ver_id_comp
: ver_sq_bicat_ver_id_comp horizontal_dual_ver_sq_bicat.
Proof.
repeat split ; cbn.
- exact (Ξ» (x : B), id_v x).
- exact (Ξ» (x y z : B)
(vβ : x -|-> y) (vβ : y -|-> z),
vβ Β· vβ).
- exact (Ξ» (x y : B)
(vβ vβ : x -|-> y),
vβ =|=> vβ).
Defined.
Definition horizontal_dual_ver_sq_bicat_id_comp_cells
: ver_sq_bicat_id_comp_cells horizontal_dual_ver_sq_bicat_ver_id_comp.
Proof.
repeat split ; cbn.
- exact (Ξ» (x y : B) (v : x -|-> y), id2 v).
- exact (Ξ» (x y : B) (v : x -|-> y), lunitor (C := op2_bicat π) v).
- exact (Ξ» (x y : B) (v : x -|-> y), runitor (C := op2_bicat π) v).
- exact (Ξ» (x y : B) (v : x -|-> y), linvunitor (C := op2_bicat π) v).
- exact (Ξ» (x y : B) (v : x -|-> y), rinvunitor (C := op2_bicat π) v).
- exact (Ξ» (w x y z : B)
(vβ : w -|-> x) (vβ : x -|-> y) (vβ : y -|-> z),
rassociator (C := op2_bicat π) vβ vβ vβ).
- exact (Ξ» (w x y z : B)
(vβ : w -|-> x) (vβ : x -|-> y) (vβ : y -|-> z),
lassociator (C := op2_bicat π) vβ vβ vβ).
- exact (Ξ» (x y : B)
(vβ vβ vβ : x -|-> y)
(Ο : vβ =|=> vβ) (ΞΈ : vβ =|=> vβ),
ΞΈ β’ Ο).
- exact (Ξ» (x y z : B)
(v : x -|-> y)
(wβ wβ : y -|-> z)
(Ο : wβ =|=> wβ),
v β Ο).
- exact (Ξ» (x y z : B)
(vβ vβ : x -|-> y)
(w : y -|-> z)
(Ο : vβ =|=> vβ),
Ο βΉ w).
Defined.
Proposition horizontal_dual_ver_sq_bicat_prebicat_laws
: ver_sq_bicat_prebicat_laws horizontal_dual_ver_sq_bicat_id_comp_cells.
Proof.
exact (pr21 (op2_bicat π)).
Qed.
Definition horizontal_dual_ver_bicat_sq_bicat
: ver_bicat_sq_bicat.
Proof.
use make_ver_bicat_sq_bicat.
- exact horizontal_dual_ver_sq_bicat.
- exact horizontal_dual_ver_sq_bicat_ver_id_comp.
- exact horizontal_dual_ver_sq_bicat_id_comp_cells.
- exact horizontal_dual_ver_sq_bicat_prebicat_laws.
- abstract
(intro ; intros ;
apply cellset_property).
Defined.
Definition horizontal_dual_ver_bicat_sq_bicat_ver_id_comp_sq
: ver_bicat_sq_bicat_ver_id_comp_sq horizontal_dual_ver_bicat_sq_bicat.
Proof.
split.
- exact (Ξ» (x y : B) (h : y --> x), id_v_square_bicat h).
- exact (Ξ» (xβ xβ xβ yβ yβ yβ : B)
(hβ : yβ --> xβ)
(hβ : yβ --> xβ)
(hβ : yβ --> xβ)
(vβ : xβ -|-> xβ) (vβ : xβ -|-> xβ)
(wβ : yβ -|-> yβ) (wβ : yβ -|-> yβ)
(sβ : square_double_bicat hβ hβ wβ vβ)
(sβ : square_double_bicat hβ hβ wβ vβ),
sβ βv sβ).
Defined.
Definition horizontal_dual_ver_bicat_sq_bicat_ver_id_comp
: ver_bicat_sq_bicat_ver_id_comp.
Proof.
use make_ver_bicat_sq_bicat_ver_id_comp.
- exact horizontal_dual_ver_bicat_sq_bicat.
- exact horizontal_dual_ver_bicat_sq_bicat_ver_id_comp_sq.
Defined.
: bicat
:= op1_bicat (hor_bicat_of_verity_double_bicat B).
Definition horizontal_dual_twosided_disp_cat_data
: twosided_disp_cat_data horizontal_dual_hor_bicat horizontal_dual_hor_bicat.
Proof.
simple refine ((_ ,, _) ,, (_ ,, _)).
- exact (Ξ» (x y : B), x -|-> y).
- exact (Ξ» (xβ xβ yβ yβ : B)
(vβ : xβ -|-> yβ) (vβ : xβ -|-> yβ)
(hβ : xβ --> xβ) (hβ : yβ --> yβ),
square_double_bicat hβ hβ vβ vβ).
- exact (Ξ» (x y : B) (v : x -|-> y), id_h_square_bicat _).
- exact (Ξ» (xβ xβ xβ yβ yβ yβ : B)
(vβ : xβ -|-> yβ) (vβ : xβ -|-> yβ) (vβ : xβ -|-> yβ)
(hβ : xβ --> xβ) (hβ : xβ --> xβ)
(kβ : yβ --> yβ) (kβ : yβ --> yβ)
(sβ : square_double_bicat hβ kβ vβ vβ)
(sβ : square_double_bicat hβ kβ vβ vβ),
sβ βh sβ).
Defined.
Definition horizontal_dual_ver_sq_bicat
: ver_sq_bicat.
Proof.
use make_ver_sq_bicat.
- exact horizontal_dual_hor_bicat.
- exact horizontal_dual_twosided_disp_cat_data.
Defined.
Definition horizontal_dual_ver_sq_bicat_ver_id_comp
: ver_sq_bicat_ver_id_comp horizontal_dual_ver_sq_bicat.
Proof.
repeat split ; cbn.
- exact (Ξ» (x : B), id_v x).
- exact (Ξ» (x y z : B)
(vβ : x -|-> y) (vβ : y -|-> z),
vβ Β· vβ).
- exact (Ξ» (x y : B)
(vβ vβ : x -|-> y),
vβ =|=> vβ).
Defined.
Definition horizontal_dual_ver_sq_bicat_id_comp_cells
: ver_sq_bicat_id_comp_cells horizontal_dual_ver_sq_bicat_ver_id_comp.
Proof.
repeat split ; cbn.
- exact (Ξ» (x y : B) (v : x -|-> y), id2 v).
- exact (Ξ» (x y : B) (v : x -|-> y), lunitor (C := op2_bicat π) v).
- exact (Ξ» (x y : B) (v : x -|-> y), runitor (C := op2_bicat π) v).
- exact (Ξ» (x y : B) (v : x -|-> y), linvunitor (C := op2_bicat π) v).
- exact (Ξ» (x y : B) (v : x -|-> y), rinvunitor (C := op2_bicat π) v).
- exact (Ξ» (w x y z : B)
(vβ : w -|-> x) (vβ : x -|-> y) (vβ : y -|-> z),
rassociator (C := op2_bicat π) vβ vβ vβ).
- exact (Ξ» (w x y z : B)
(vβ : w -|-> x) (vβ : x -|-> y) (vβ : y -|-> z),
lassociator (C := op2_bicat π) vβ vβ vβ).
- exact (Ξ» (x y : B)
(vβ vβ vβ : x -|-> y)
(Ο : vβ =|=> vβ) (ΞΈ : vβ =|=> vβ),
ΞΈ β’ Ο).
- exact (Ξ» (x y z : B)
(v : x -|-> y)
(wβ wβ : y -|-> z)
(Ο : wβ =|=> wβ),
v β Ο).
- exact (Ξ» (x y z : B)
(vβ vβ : x -|-> y)
(w : y -|-> z)
(Ο : vβ =|=> vβ),
Ο βΉ w).
Defined.
Proposition horizontal_dual_ver_sq_bicat_prebicat_laws
: ver_sq_bicat_prebicat_laws horizontal_dual_ver_sq_bicat_id_comp_cells.
Proof.
exact (pr21 (op2_bicat π)).
Qed.
Definition horizontal_dual_ver_bicat_sq_bicat
: ver_bicat_sq_bicat.
Proof.
use make_ver_bicat_sq_bicat.
- exact horizontal_dual_ver_sq_bicat.
- exact horizontal_dual_ver_sq_bicat_ver_id_comp.
- exact horizontal_dual_ver_sq_bicat_id_comp_cells.
- exact horizontal_dual_ver_sq_bicat_prebicat_laws.
- abstract
(intro ; intros ;
apply cellset_property).
Defined.
Definition horizontal_dual_ver_bicat_sq_bicat_ver_id_comp_sq
: ver_bicat_sq_bicat_ver_id_comp_sq horizontal_dual_ver_bicat_sq_bicat.
Proof.
split.
- exact (Ξ» (x y : B) (h : y --> x), id_v_square_bicat h).
- exact (Ξ» (xβ xβ xβ yβ yβ yβ : B)
(hβ : yβ --> xβ)
(hβ : yβ --> xβ)
(hβ : yβ --> xβ)
(vβ : xβ -|-> xβ) (vβ : xβ -|-> xβ)
(wβ : yβ -|-> yβ) (wβ : yβ -|-> yβ)
(sβ : square_double_bicat hβ hβ wβ vβ)
(sβ : square_double_bicat hβ hβ wβ vβ),
sβ βv sβ).
Defined.
Definition horizontal_dual_ver_bicat_sq_bicat_ver_id_comp
: ver_bicat_sq_bicat_ver_id_comp.
Proof.
use make_ver_bicat_sq_bicat_ver_id_comp.
- exact horizontal_dual_ver_bicat_sq_bicat.
- exact horizontal_dual_ver_bicat_sq_bicat_ver_id_comp_sq.
Defined.
Definition horizontal_dual_double_bicat_whiskering
: double_bicat_whiskering horizontal_dual_ver_bicat_sq_bicat_ver_id_comp.
Proof.
repeat split.
- exact (Ξ» (w x y z : B)
(hβ : x --> w)
(hβ : z --> y)
(vβ vβ' : w -|-> y)
(vβ : x -|-> z)
(Ο : vβ' =|=> vβ)
(s : square_double_bicat hβ hβ vβ vβ'),
Ο βΉs s).
- exact (Ξ» (w x y z : B)
(hβ : x --> w)
(hβ : z --> y)
(vβ : w -|-> y)
(vβ vβ' : x -|-> z)
(Ο : vβ' =|=> vβ)
(s : square_double_bicat hβ hβ vβ vβ),
Ο βs s).
- exact (Ξ» (w x y z : B)
(hβ hβ' : x --> w)
(hβ : z --> y)
(vβ : w -|-> y)
(vβ : x -|-> z)
(Ο : hβ ==> hβ')
(s : square_double_bicat hβ' hβ vβ vβ),
Ο β΅s s).
- exact (Ξ» (w x y z : B)
(hβ : x --> w)
(hβ hβ' : z --> y)
(vβ : w -|-> y)
(vβ : x -|-> z)
(Ο : hβ ==> hβ')
(s : square_double_bicat hβ hβ vβ vβ),
Ο βΏs s).
Defined.
Definition horizontal_dual_ver_bicat_sq_id_comp_whisker
: ver_bicat_sq_id_comp_whisker.
Proof.
use make_ver_bicat_sq_id_comp_whisker.
- exact horizontal_dual_ver_bicat_sq_bicat_ver_id_comp.
- exact horizontal_dual_double_bicat_whiskering.
Defined.
: double_bicat_whiskering horizontal_dual_ver_bicat_sq_bicat_ver_id_comp.
Proof.
repeat split.
- exact (Ξ» (w x y z : B)
(hβ : x --> w)
(hβ : z --> y)
(vβ vβ' : w -|-> y)
(vβ : x -|-> z)
(Ο : vβ' =|=> vβ)
(s : square_double_bicat hβ hβ vβ vβ'),
Ο βΉs s).
- exact (Ξ» (w x y z : B)
(hβ : x --> w)
(hβ : z --> y)
(vβ : w -|-> y)
(vβ vβ' : x -|-> z)
(Ο : vβ' =|=> vβ)
(s : square_double_bicat hβ hβ vβ vβ),
Ο βs s).
- exact (Ξ» (w x y z : B)
(hβ hβ' : x --> w)
(hβ : z --> y)
(vβ : w -|-> y)
(vβ : x -|-> z)
(Ο : hβ ==> hβ')
(s : square_double_bicat hβ' hβ vβ vβ),
Ο β΅s s).
- exact (Ξ» (w x y z : B)
(hβ : x --> w)
(hβ hβ' : z --> y)
(vβ : w -|-> y)
(vβ : x -|-> z)
(Ο : hβ ==> hβ')
(s : square_double_bicat hβ hβ vβ vβ),
Ο βΏs s).
Defined.
Definition horizontal_dual_ver_bicat_sq_id_comp_whisker
: ver_bicat_sq_id_comp_whisker.
Proof.
use make_ver_bicat_sq_id_comp_whisker.
- exact horizontal_dual_ver_bicat_sq_bicat_ver_id_comp.
- exact horizontal_dual_double_bicat_whiskering.
Defined.
Proposition horizontal_dual_whisker_square_bicat_law
: whisker_square_bicat_law horizontal_dual_ver_bicat_sq_id_comp_whisker.
Proof.
repeat split ; intro ; intros ; cbn.
- apply rwhisker_square_id.
- apply rwhisker_square_comp.
- apply lwhisker_square_id.
- apply lwhisker_square_comp.
- apply uwhisker_square_id.
- apply uwhisker_square_comp.
- apply dwhisker_square_id.
- apply dwhisker_square_comp.
- apply dwhisker_uwhisker_square.
- apply rwhisker_uwhisker_square.
- apply lwhisker_uwhisker_square.
- apply rwhisker_dwhisker_square.
- apply lwhisker_dwhisker_square.
- refine (!_).
apply rwhisker_lwhisker_square.
- refine (!_).
apply lwhisker_id_h_square.
- apply uwhisker_id_v_square.
- apply uwhisker_vcomp_square.
- apply dwhisker_vcomp_square.
- apply ud_whisker_vcomp_square.
- apply rwhisker_hcomp_square.
- apply lwhisker_hcomp_square.
- refine (!_).
apply lrwhisker_hcomp_square.
Qed.
Proposition horizontal_dual_double_bicat_id_comp_square_laws
: double_bicat_id_comp_square_laws horizontal_dual_ver_bicat_sq_id_comp_whisker.
Proof.
repeat split ; intro ; intros ; cbn.
- apply double_bicat_interchange.
- apply id_h_square_bicat_id.
- apply id_h_square_bicat_comp.
- apply id_v_square_bicat_comp.
Qed.
Proposition horizontal_dual_double_bicat_cylinder_laws
: double_bicat_cylinder_laws horizontal_dual_ver_bicat_sq_id_comp_whisker.
Proof.
repeat split.
- intro ; intros ; cbn.
etrans.
{
apply maponpaths.
apply lassociator_h_comp_square''.
}
rewrite <- dwhisker_square_comp.
rewrite lassociator_rassociator.
apply dwhisker_square_id.
- intro ; intros ; cbn.
etrans.
{
apply maponpaths.
apply lassociator_v_comp_square'.
}
rewrite <- rwhisker_lwhisker_square.
rewrite <- rwhisker_square_comp.
rewrite (lassociator_rassociator (C := π)).
apply rwhisker_square_id.
- intro ; intros ; cbn.
apply runitor_h_comp_square.
- intro ; intros ; cbn.
refine (!_).
etrans.
{
apply maponpaths.
apply lunitor_v_comp_square'.
}
rewrite rwhisker_lwhisker_square.
rewrite <- lwhisker_square_comp.
rewrite (linvunitor_lunitor (C := π)).
apply lwhisker_square_id.
- intro ; intros ; cbn.
apply lunitor_h_comp_square.
- intro ; intros ; cbn.
refine (!_).
etrans.
{
apply maponpaths.
apply runitor_v_comp_square'.
}
rewrite rwhisker_lwhisker_square.
rewrite <- lwhisker_square_comp.
rewrite (rinvunitor_runitor (C := π)).
apply lwhisker_square_id.
- intros xβ xβ yβ yβ zβ zβ hβ hβ hβ vβ vβ' vβ vβ'.
intros wβ wβ' wβ wβ' Οβ Οβ ΞΈβ ΞΈβ sβ sβ' sβ sβ' p q ; cbn.
rewrite <- !(vcomp_whisker (C := π)).
exact (!(ver_bicat_hcomp_v_comp_square B _ _ _ _ _ _ _ _ (!p) (!q))).
- intros xβ xβ yβ yβ zβ zβ hβ hβ hβ vβ vβ' vβ vβ'.
intros wβ wβ' wβ wβ' Οβ Οβ ΞΈβ ΞΈβ sβ sβ' sβ sβ' p q ; cbn.
rewrite <- !vcomp_whisker.
exact (hor_bicat_hcomp_h_comp_square B _ _ _ _ _ _ _ _ q p).
Qed.
Proposition horizontal_dual_double_bicat_laws
: double_bicat_laws horizontal_dual_ver_bicat_sq_id_comp_whisker.
Proof.
use make_double_bicat_laws.
- exact horizontal_dual_whisker_square_bicat_law.
- exact horizontal_dual_double_bicat_id_comp_square_laws.
- exact horizontal_dual_double_bicat_cylinder_laws.
- intro ; intros.
apply isaset_square_double_bicat.
Qed.
: whisker_square_bicat_law horizontal_dual_ver_bicat_sq_id_comp_whisker.
Proof.
repeat split ; intro ; intros ; cbn.
- apply rwhisker_square_id.
- apply rwhisker_square_comp.
- apply lwhisker_square_id.
- apply lwhisker_square_comp.
- apply uwhisker_square_id.
- apply uwhisker_square_comp.
- apply dwhisker_square_id.
- apply dwhisker_square_comp.
- apply dwhisker_uwhisker_square.
- apply rwhisker_uwhisker_square.
- apply lwhisker_uwhisker_square.
- apply rwhisker_dwhisker_square.
- apply lwhisker_dwhisker_square.
- refine (!_).
apply rwhisker_lwhisker_square.
- refine (!_).
apply lwhisker_id_h_square.
- apply uwhisker_id_v_square.
- apply uwhisker_vcomp_square.
- apply dwhisker_vcomp_square.
- apply ud_whisker_vcomp_square.
- apply rwhisker_hcomp_square.
- apply lwhisker_hcomp_square.
- refine (!_).
apply lrwhisker_hcomp_square.
Qed.
Proposition horizontal_dual_double_bicat_id_comp_square_laws
: double_bicat_id_comp_square_laws horizontal_dual_ver_bicat_sq_id_comp_whisker.
Proof.
repeat split ; intro ; intros ; cbn.
- apply double_bicat_interchange.
- apply id_h_square_bicat_id.
- apply id_h_square_bicat_comp.
- apply id_v_square_bicat_comp.
Qed.
Proposition horizontal_dual_double_bicat_cylinder_laws
: double_bicat_cylinder_laws horizontal_dual_ver_bicat_sq_id_comp_whisker.
Proof.
repeat split.
- intro ; intros ; cbn.
etrans.
{
apply maponpaths.
apply lassociator_h_comp_square''.
}
rewrite <- dwhisker_square_comp.
rewrite lassociator_rassociator.
apply dwhisker_square_id.
- intro ; intros ; cbn.
etrans.
{
apply maponpaths.
apply lassociator_v_comp_square'.
}
rewrite <- rwhisker_lwhisker_square.
rewrite <- rwhisker_square_comp.
rewrite (lassociator_rassociator (C := π)).
apply rwhisker_square_id.
- intro ; intros ; cbn.
apply runitor_h_comp_square.
- intro ; intros ; cbn.
refine (!_).
etrans.
{
apply maponpaths.
apply lunitor_v_comp_square'.
}
rewrite rwhisker_lwhisker_square.
rewrite <- lwhisker_square_comp.
rewrite (linvunitor_lunitor (C := π)).
apply lwhisker_square_id.
- intro ; intros ; cbn.
apply lunitor_h_comp_square.
- intro ; intros ; cbn.
refine (!_).
etrans.
{
apply maponpaths.
apply runitor_v_comp_square'.
}
rewrite rwhisker_lwhisker_square.
rewrite <- lwhisker_square_comp.
rewrite (rinvunitor_runitor (C := π)).
apply lwhisker_square_id.
- intros xβ xβ yβ yβ zβ zβ hβ hβ hβ vβ vβ' vβ vβ'.
intros wβ wβ' wβ wβ' Οβ Οβ ΞΈβ ΞΈβ sβ sβ' sβ sβ' p q ; cbn.
rewrite <- !(vcomp_whisker (C := π)).
exact (!(ver_bicat_hcomp_v_comp_square B _ _ _ _ _ _ _ _ (!p) (!q))).
- intros xβ xβ yβ yβ zβ zβ hβ hβ hβ vβ vβ' vβ vβ'.
intros wβ wβ' wβ wβ' Οβ Οβ ΞΈβ ΞΈβ sβ sβ' sβ sβ' p q ; cbn.
rewrite <- !vcomp_whisker.
exact (hor_bicat_hcomp_h_comp_square B _ _ _ _ _ _ _ _ q p).
Qed.
Proposition horizontal_dual_double_bicat_laws
: double_bicat_laws horizontal_dual_ver_bicat_sq_id_comp_whisker.
Proof.
use make_double_bicat_laws.
- exact horizontal_dual_whisker_square_bicat_law.
- exact horizontal_dual_double_bicat_id_comp_square_laws.
- exact horizontal_dual_double_bicat_cylinder_laws.
- intro ; intros.
apply isaset_square_double_bicat.
Qed.
Definition horizontal_dual_verity_double_bicat
: verity_double_bicat.
Proof.
use make_verity_double_bicat.
- exact horizontal_dual_ver_bicat_sq_id_comp_whisker.
- exact horizontal_dual_double_bicat_laws.
Defined.
: verity_double_bicat.
Proof.
use make_verity_double_bicat.
- exact horizontal_dual_ver_bicat_sq_id_comp_whisker.
- exact horizontal_dual_double_bicat_laws.
Defined.
Definition horizontal_dual_vertically_saturated
(H : vertically_saturated B)
: vertically_saturated horizontal_dual_verity_double_bicat.
Proof.
refine (Ξ» (x y : B) (vβ vβ : x -|-> y), _).
use isweq_iso.
- exact (Ξ» s, square_to_vertical_cell H s).
- abstract
(intro Ο ; cbn ;
refine (_ @ vertical_cell_to_square_to_vertical_cell H Ο) ;
apply maponpaths ; unfold vertical_cell_to_square ;
rewrite lwhisker_id_h_square ;
apply idpath).
- abstract
(intro s ; cbn ;
refine (_ @ square_to_vertical_cell_to_square H s) ;
unfold vertical_cell_to_square ;
rewrite lwhisker_id_h_square ;
apply idpath).
Defined.
(H : vertically_saturated B)
: vertically_saturated horizontal_dual_verity_double_bicat.
Proof.
refine (Ξ» (x y : B) (vβ vβ : x -|-> y), _).
use isweq_iso.
- exact (Ξ» s, square_to_vertical_cell H s).
- abstract
(intro Ο ; cbn ;
refine (_ @ vertical_cell_to_square_to_vertical_cell H Ο) ;
apply maponpaths ; unfold vertical_cell_to_square ;
rewrite lwhisker_id_h_square ;
apply idpath).
- abstract
(intro s ; cbn ;
refine (_ @ square_to_vertical_cell_to_square H s) ;
unfold vertical_cell_to_square ;
rewrite lwhisker_id_h_square ;
apply idpath).
Defined.
Proposition hor_locally_univalent_horizontal_dual
(H : hor_locally_univalent B)
: hor_locally_univalent horizontal_dual_verity_double_bicat.
Proof.
use op1_bicat_is_univalent_2_1.
exact H.
Qed.
Definition horizontal_dual_inv2cell_weq
{x y : B}
(vβ vβ : x -|-> y)
: invertible_2cell (C := π) vβ vβ
β
invertible_2cell
(C := ver_bicat_of_verity_double_bicat horizontal_dual_verity_double_bicat)
vβ vβ.
Proof.
use weq_iso.
- use (Ξ» Ο, make_invertible_2cell _).
+ exact Ο^-1.
+ use make_is_invertible_2cell.
* exact Ο.
* exact (vcomp_rinv Ο).
* exact (vcomp_linv Ο).
- use (Ξ» Ο, make_invertible_2cell _).
+ exact Ο^-1.
+ use make_is_invertible_2cell.
* exact Ο.
* exact (vcomp_rinv Ο).
* exact (vcomp_linv Ο).
- abstract
(intro ;
apply idpath).
- abstract
(intro ;
apply idpath).
Defined.
Proposition ver_locally_univalent_horizontal_dual
(H : ver_locally_univalent B)
: ver_locally_univalent horizontal_dual_verity_double_bicat.
Proof.
intros x y vβ vβ.
use weqhomot.
- exact (horizontal_dual_inv2cell_weq vβ vβ
β make_weq _ (H x y vβ vβ))%weq.
- intro p.
induction p.
use cell_from_invertible_2cell_eq ; cbn.
apply idpath.
Qed.
Proposition locally_univalent_horizontal_dual
(H : locally_univalent_verity_double_bicat B)
: locally_univalent_verity_double_bicat horizontal_dual_verity_double_bicat.
Proof.
split.
- use hor_locally_univalent_horizontal_dual.
apply H.
- use ver_locally_univalent_horizontal_dual.
apply H.
Qed.
End HorizontalDual.
(H : hor_locally_univalent B)
: hor_locally_univalent horizontal_dual_verity_double_bicat.
Proof.
use op1_bicat_is_univalent_2_1.
exact H.
Qed.
Definition horizontal_dual_inv2cell_weq
{x y : B}
(vβ vβ : x -|-> y)
: invertible_2cell (C := π) vβ vβ
β
invertible_2cell
(C := ver_bicat_of_verity_double_bicat horizontal_dual_verity_double_bicat)
vβ vβ.
Proof.
use weq_iso.
- use (Ξ» Ο, make_invertible_2cell _).
+ exact Ο^-1.
+ use make_is_invertible_2cell.
* exact Ο.
* exact (vcomp_rinv Ο).
* exact (vcomp_linv Ο).
- use (Ξ» Ο, make_invertible_2cell _).
+ exact Ο^-1.
+ use make_is_invertible_2cell.
* exact Ο.
* exact (vcomp_rinv Ο).
* exact (vcomp_linv Ο).
- abstract
(intro ;
apply idpath).
- abstract
(intro ;
apply idpath).
Defined.
Proposition ver_locally_univalent_horizontal_dual
(H : ver_locally_univalent B)
: ver_locally_univalent horizontal_dual_verity_double_bicat.
Proof.
intros x y vβ vβ.
use weqhomot.
- exact (horizontal_dual_inv2cell_weq vβ vβ
β make_weq _ (H x y vβ vβ))%weq.
- intro p.
induction p.
use cell_from_invertible_2cell_eq ; cbn.
apply idpath.
Qed.
Proposition locally_univalent_horizontal_dual
(H : locally_univalent_verity_double_bicat B)
: locally_univalent_verity_double_bicat horizontal_dual_verity_double_bicat.
Proof.
split.
- use hor_locally_univalent_horizontal_dual.
apply H.
- use ver_locally_univalent_horizontal_dual.
apply H.
Qed.
End HorizontalDual.