------------------------------------------------------------------------
-- The Agda standard library
--
-- Some properties imply others
------------------------------------------------------------------------

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

module Relation.Unary.Consequences where

open import Relation.Unary
open import Relation.Nullary using (recompute)

dec⟶recomputable : {a  : _} {A : Set a} {P : Pred A }  Decidable P  Recomputable P
dec⟶recomputable P-dec = recompute (P-dec _)