summaryrefslogtreecommitdiff
path: root/src/Data/Star.agda
blob: 00f1f5ac667f1d38c9536130c796e39e86ec35bd (plain)
1
2
3
4
5
6
7
8
9
10
11
12
------------------------------------------------------------------------
-- The Agda standard library
--
-- The reflexive transitive closures of McBride, Norell and Jansson
--
-- This module is DEPRECATED. Please use the
-- Relation.Binary.Construct.Closure.ReflexiveTransitive module directly
------------------------------------------------------------------------

module Data.Star where

open import Relation.Binary.Construct.Closure.ReflexiveTransitive public