mirror of
https://git8.cs.fau.de/theses/bsc-leon-vatthauer.git
synced 2024-05-31 07:28:34 +02:00
31 lines
874 B
Agda
31 lines
874 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
|
||
open import Distributive.Core
|
||
open import Extensive.Core
|
||
import Categories.Morphism as M
|
||
|
||
module Extensive.Bundle where
|
||
|
||
open import Level
|
||
|
||
record ExtensiveCategory o ℓ e : Set (suc (o ⊔ ℓ ⊔ e)) where
|
||
field
|
||
U : Category o ℓ e
|
||
extensive : Extensive U
|
||
|
||
open Category U public
|
||
open Extensive extensive public
|
||
|
||
record ExtensiveDistributiveCategory o ℓ e : Set (suc (o ⊔ ℓ ⊔ e)) where
|
||
field
|
||
U : Category o ℓ e
|
||
cartesian : Cartesian U
|
||
extensive : Extensive U
|
||
|
||
open Category U public
|
||
open Extensive extensive public
|
||
open Distributive (Extensive⇒Distributive cartesian extensive) public
|