module WellFoundedTree where

open import Level

infix 1 W
data W { ℓ' : Level}(A : Set )(B : A  Set ℓ') : Set (  ℓ') where
  sup : (x : A)(f : B x  W A B)  W A B

syntax W A  x  B) = W x ∈ A , B