{-# OPTIONS --cubical-compatible --safe #-}
module Function.Properties.Injection where
open import Function.Base
open import Function.Definitions
open import Function.Bundles
import Function.Construct.Identity as Identity
import Function.Construct.Composition as Compose
open import Level using (Level)
open import Data.Product.Base using (proj₁; proj₂)
open import Relation.Binary.Definitions
open import Relation.Binary.PropositionalEquality using ()
open import Relation.Binary using (Setoid)
import Relation.Binary.Reasoning.Setoid as SetoidReasoning
private
  variable
    a b c ℓ ℓ₁ ℓ₂ ℓ₃ : Level
    A B : Set a
    T S U : Setoid a ℓ
mkInjection : (f : Func S T) (open Func f) →
              Injective Eq₁._≈_ Eq₂._≈_ to  →
              Injection S T
mkInjection f injective = record
  { Func f
  ; injective = injective
  }
↣⇒⟶ : A ↣ B → A ⟶ B
↣⇒⟶ = Injection.function
refl : Reflexive (Injection {a} {ℓ})
refl {x = x} = Identity.injection x
trans : Trans (Injection {a} {ℓ₁} {b} {ℓ₂})
              (Injection {b} {ℓ₂} {c} {ℓ₃})
              (Injection {a} {ℓ₁} {c} {ℓ₃})
trans = Compose.injection
↣-refl : Injection S S
↣-refl = refl
↣-trans : Injection S T → Injection T U → Injection S U
↣-trans = trans