aboutsummaryrefslogtreecommitdiff
path: root/Data/Hypergraph.agda
blob: 2e8498cc9205537c79f85de8b73e2d131cf0f88e (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
{-# OPTIONS --without-K --safe #-}

open import Level using (Level)

open import Data.Hypergraph.Label using (HypergraphLabel)

module Data.Hypergraph {c  : Level} (HL : HypergraphLabel) where

open import Data.Hypergraph.Base {c} HL public
open import Data.Hypergraph.Setoid {c} {} HL public

import Data.Hypergraph.Edge HL as HypergraphEdge

module Edge = HypergraphEdge