Skip to content

Commit

Permalink
Merge pull request #5 from Olavhaasie/fix-bundles
Browse files Browse the repository at this point in the history
Fix bundles
  • Loading branch information
ajrouvoet authored Jan 28, 2022
2 parents 4bad4cf + 7458ddb commit fe131ce
Showing 1 changed file with 12 additions and 12 deletions.
24 changes: 12 additions & 12 deletions src/Relation/Ternary/Bundles.agda
Original file line number Diff line number Diff line change
@@ -1,12 +1,13 @@
{-# OPTIONS --postfix-projections #-}
{-# OPTIONS --safe --without-K #-}
module Relation.Ternary.Bundles where

open import Level
open import Relation.Binary
open import Relation.Binary.Bundles
open import Relation.Ternary.Core hiding (_✴_)
open import Relation.Ternary.Core
open import Relation.Ternary.Structures using
( IsPartialSemigroup
( Emptiness
; IsPartialSemigroup
; IsPartialMonoid
; IsJoinoid )

Expand All @@ -33,20 +34,19 @@ record PartialSemigroup a e : Set (suc (a ⊔ e)) where

record PartialMonoid a e : Set (suc (a ⊔ e)) where
field
{Carrier} : Set a
{_≈_} : Carrier Carrier Set e
{rel} : Rel₃ Carrier
{unit} : Carrier
{Carrier} : Set a
{_≈_} : Carrier Carrier Set e
{rel} : Rel₃ Carrier
{unit} : Carrier

isMonoid : IsPartialMonoid _≈_ rel unit
isMonoid : IsPartialMonoid _≈_ rel unit

open IsPartialMonoid isMonoid public
open Emptiness emptiness public
open IsPartialSemigroup isSemigroup public

instance partialSemigroup : PartialSemigroup a e
partialSemigroup = record { isSemigroup = isPartialSemigroup }

open PartialSemigroup {{...}} public
open PartialMonoid {{...}} public
partialSemigroup = record { isSemigroup = isSemigroup }

-- record PartialJoinoid a e : Set (suc (a ⊔ e)) where
-- field
Expand Down

0 comments on commit fe131ce

Please sign in to comment.