------------------------------------------------------------------------
-- The Agda standard library
--
-- Indexed unary relations
------------------------------------------------------------------------

{-# OPTIONS --cubical-compatible --safe #-}

module Relation.Unary.Indexed  where

open import Data.Product.Base using (; _×_)
open import Level
open import Relation.Nullary.Negation using (¬_)

IPred :  {i a} {I : Set i}  (I  Set a)  ( : Level)  Set _
IPred A  =  {i}  A i  Set 

module _ {i a} {I : Set i} {A : I  Set a} where

  infix 4 _∈_ _∉_

  _∈_ :  {}  (∀ i  A i)  IPred A   Set _
  x  P =  i  P (x i)

  _∉_ :  {}  (∀ i  A i)  IPred A   Set _
  t  P = ¬ (t  P)