mirror of
https://git8.cs.fau.de/theses/bsc-leon-vatthauer.git
synced 2024-05-31 07:28:34 +02:00
29 lines
777 B
Agda
29 lines
777 B
Agda
|
{-# OPTIONS --without-K --safe #-}
|
|||
|
|
|||
|
open import Categories.Category
|
|||
|
open import Categories.Category.Cartesian
|
|||
|
open import Categories.Category.BinaryProducts
|
|||
|
open import Categories.Category.Cocartesian
|
|||
|
import Categories.Morphism as M
|
|||
|
|
|||
|
module Distributive.Core {o ℓ e} (𝒞 : Category o ℓ e) where
|
|||
|
|
|||
|
open import Level
|
|||
|
open Category 𝒞
|
|||
|
open M 𝒞
|
|||
|
|
|||
|
record Distributive : Set (levelOfTerm 𝒞) where
|
|||
|
field
|
|||
|
cartesian : Cartesian 𝒞
|
|||
|
cocartesian : Cocartesian 𝒞
|
|||
|
|
|||
|
open Cartesian cartesian
|
|||
|
open BinaryProducts products
|
|||
|
open Cocartesian cocartesian
|
|||
|
|
|||
|
distribute : ∀ {A B C} → (A × B + A × C) ⇒ (A × (B + C))
|
|||
|
distribute = [ id ⁂ i₁ , id ⁂ i₂ ]
|
|||
|
|
|||
|
field
|
|||
|
iso : ∀ {A B C} → IsIso (distribute {A} {B} {C})
|