Some graphs stuff (#98)

This commit is contained in:
Patrick Stevens
2020-02-15 13:41:51 +00:00
committed by GitHub
parent 9de323c5e8
commit f41f5226b9
18 changed files with 275 additions and 39 deletions

View File

@@ -0,0 +1,23 @@
{-# OPTIONS --warning=error --safe --without-K #-}
open import LogicalFormulae
open import Agda.Primitive using (Level; lzero; lsuc; _⊔_)
open import Functions
open import Setoids.Setoids
open import Setoids.Subset
open import Graphs.Definition
open import Sets.FinSet.Definition
open import Numbers.Naturals.Semiring
open import Numbers.Naturals.Order
open import Sets.EquivalenceRelations
open import Graphs.CompleteGraph
open import Graphs.Colouring
module Graphs.RamseyTriangle where
hasMonochromaticTriangle : {a : _} {n : } (G : Graph a (reflSetoid (FinSet n))) Set (lsuc lzero)
hasMonochromaticTriangle {n = n} G = Sg (FinSet n Set) λ pred (subset (reflSetoid (FinSet n)) pred) && {!!}
ramseyForTriangle : (k : ) Sg (λ N (n : ) (N <N n) (c : Colouring k (Kn n)) {!!})
ramseyForTriangle k = {!!}