Star.agda 173 B

1234567
  1. module Star where
  2. data Star {A : Set}(R : A -> A -> Set) : A -> A -> Set where
  3. rf : {x : A} -> Star R x x
  4. _<>_ : forall {x y z} -> R x y -> Star R y z -> Star R x z