Documentation

Mathlib.Tactic.CategoryTheory.Bicategory.PureCoherence

Coherence tactic for bicategories #

We provide a bicategory_coherence tactic, which proves that any two morphisms (with the same source and target) in a bicategory which are built out of associators and unitors are equal.

@[reducible, inline]

The composition of the normalizing isomorphisms η_f : p ≫ f ≅ pf and η_g : pf ≫ g ≅ pfg.

Equations
Instances For

    Close the goal of the form η = θ, where η and θ are 2-isomorphisms made up only of associators, unitors, and identities.

    example {B : Type} [Bicategory B] {a : B} :
      (λ_ (𝟙 a)).hom = (ρ_ (𝟙 a)).hom := by
      bicategory_coherence
    
    Equations
    Instances For

      Close the goal of the form η = θ, where η and θ are 2-isomorphisms made up only of associators, unitors, and identities.

      example {B : Type} [Bicategory B] {a : B} :
        (λ_ (𝟙 a)).hom = (ρ_ (𝟙 a)).hom := by
        bicategory_coherence
      
      Equations
      • One or more equations did not get rendered due to their size.
      Instances For