Skip to content

Commit

Permalink
Prove edge-clique law
Browse files Browse the repository at this point in the history
  • Loading branch information
snowleopard committed Apr 17, 2017
1 parent 1b0651a commit e59826c
Showing 1 changed file with 4 additions and 0 deletions.
4 changes: 4 additions & 0 deletions src/API/Theorems.agda
Original file line number Diff line number Diff line change
Expand Up @@ -10,6 +10,10 @@ open import Reasoning
vertices-vertex : {A} {x : A} -> vertices [ x ] ≡ vertex x
vertices-vertex = +identity >> reflexivity

-- edge x y == clique [x, y]
edge-clique : {A} {x y : A} -> edge x y ≡ clique (x :: [ y ])
edge-clique = symmetry (R *right-identity)

-- vertices xs ⊆ clique xs
vertices-clique : {A} {xs : List A} -> vertices xs ⊆ clique xs
vertices-clique {_} {[]} = ⊆reflexivity
Expand Down

0 comments on commit e59826c

Please sign in to comment.