Skip to content
Merged
Show file tree
Hide file tree
Changes from all commits
Commits
File filter

Filter by extension

Filter by extension

Conversations
Failed to load comments.
Loading
Jump to
Jump to file
Failed to load files.
Loading
Diff view
Diff view
5 changes: 5 additions & 0 deletions src/Function/Bijection.agda
Original file line number Diff line number Diff line change
Expand Up @@ -6,6 +6,11 @@

{-# OPTIONS --without-K --safe #-}

-- Note: use of the standard function hierarchy is encouraged. The
-- module `Function` re-exports `Bijective`, `IsBijection` and
-- `Bijection`. The alternative definitions found in this file will
-- eventually be deprecated.

module Function.Bijection where

open import Data.Product
Expand Down
5 changes: 5 additions & 0 deletions src/Function/Equality.agda
Original file line number Diff line number Diff line change
Expand Up @@ -6,6 +6,11 @@

{-# OPTIONS --without-K --safe #-}

-- Note: use of the standard function hierarchy is encouraged. The
-- module `Function` re-exports `Congruent`, `IsBijection` and
-- `Bijection`. The alternative definitions found in this file will
-- eventually be deprecated.

module Function.Equality where

import Function.Base as Fun
Expand Down
7 changes: 6 additions & 1 deletion src/Function/Equivalence.agda
Original file line number Diff line number Diff line change
Expand Up @@ -8,7 +8,12 @@

module Function.Equivalence where

open import Function using (flip)
-- Note: use of the standard function hierarchy is encouraged. The
-- module `Function` re-exports `Congruent` and `IsCongruent`.
-- The alternative definitions found in this file will eventually be
-- deprecated.

open import Function.Base using (flip)
open import Function.Equality as F
using (_⟶_; _⟨$⟩_) renaming (_∘_ to _⟪∘⟫_)
open import Level
Expand Down
5 changes: 5 additions & 0 deletions src/Function/Injection.agda
Original file line number Diff line number Diff line change
Expand Up @@ -6,6 +6,11 @@

{-# OPTIONS --without-K --safe #-}

-- Note: use of the standard function hierarchy is encouraged. The
-- module `Function` re-exports `Injective`, `IsInjection` and
-- `Injection`. The alternative definitions found in this file will
-- eventually be deprecated.

module Function.Injection where

open import Function as Fun using () renaming (_∘_ to _⟨∘⟩_)
Expand Down
5 changes: 5 additions & 0 deletions src/Function/Inverse.agda
Original file line number Diff line number Diff line change
Expand Up @@ -6,6 +6,11 @@

{-# OPTIONS --without-K --safe #-}

-- Note: use of the standard function hierarchy is encouraged. The
-- module `Function` re-exports `Inverseᵇ`, `IsInverse` and
-- `Inverse`. The alternative definitions found in this file will
-- eventually be deprecated.

module Function.Inverse where

open import Level
Expand Down
5 changes: 5 additions & 0 deletions src/Function/LeftInverse.agda
Original file line number Diff line number Diff line change
Expand Up @@ -6,6 +6,11 @@

{-# OPTIONS --without-K --safe #-}

-- Note: use of the standard function hierarchy is encouraged. The
-- module `Function` re-exports `Inverseˡ`, `IsLeftInverse` and
-- `LeftInverse`. The alternative definitions found in this file will
-- eventually be deprecated.

module Function.LeftInverse where

open import Data.Product
Expand Down
5 changes: 5 additions & 0 deletions src/Function/Surjection.agda
Original file line number Diff line number Diff line change
Expand Up @@ -6,6 +6,11 @@

{-# OPTIONS --without-K --safe #-}

-- Note: use of the standard function hierarchy is encouraged. The
-- module `Function` re-exports `Surjective`, `IsSurjection` and
-- `Surjection`. The alternative definitions found in this file will
-- eventually be deprecated.

module Function.Surjection where

open import Level
Expand Down