Skip to content

Commit

Permalink
Minor fixes
Browse files Browse the repository at this point in the history
  • Loading branch information
snowleopard committed Apr 16, 2017
1 parent 3f27510 commit 9f73b5d
Showing 1 changed file with 2 additions and 3 deletions.
5 changes: 2 additions & 3 deletions src/Graph.agda
Original file line number Diff line number Diff line change
@@ -1,9 +1,9 @@
module Graph (V : Set) where
module Graph (A : Set) where

-- Core graph construction primitives
data Graph : Set where
ε : Graph -- Empty graph
[_] : V -> Graph -- Graph comprising a single vertex
[_] : A -> Graph -- Graph comprising a single vertex
_+_ : Graph -> Graph -> Graph -- Overlay two graphs
_*_ : Graph -> Graph -> Graph -- Connect two graphs

Expand Down Expand Up @@ -57,4 +57,3 @@ L {connect} {x} {y} {z} eq = *left-congruence {x} {y} {z} eq
R : {op : BinaryOperator} -> {x y z} -> x ≡ y -> apply op z x ≡ apply op z y
R {overlay} {x} {y} {z} eq = +right-congruence {x} {y} {z} eq
R {connect} {x} {y} {z} eq = *right-congruence {x} {y} {z} eq

0 comments on commit 9f73b5d

Please sign in to comment.