--------------------------------------------------------------------------------
title:          Properties of continuous maps
author:         Ayberk Tosun
date-started:   2024-04-10
--------------------------------------------------------------------------------

Factored out from the `Locales.Frame` module on 2024-04-10.

\begin{code}[hide]

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

open import MLTT.Spartan hiding (šŸš; ā‚€; ā‚)
open import UF.FunExt
open import UF.PropTrunc

module Locales.ContinuousMap.Properties
        (pt : propositional-truncations-exist)
        (fe : Fun-Ext)
       where

open import Locales.Frame pt fe
open import Locales.ContinuousMap.FrameHomomorphism-Properties pt fe
open import Locales.ContinuousMap.Definition pt fe
open import UF.Logic

open AllCombinators pt fe
open ContinuousMaps
open FrameHomomorphismProperties
open Locale

\end{code}

Lemma for showing equality of continuous maps.

\begin{code}

to-continuous-map-ļ¼ : (X : Locale š“¤ š“„ š“¦) (Y : Locale š“¤' š“„' š“¦) (f g : X ā”€cā†’ Y)
                     ā†’
                       let
                        open ContinuousMapNotation X Y
                       in
                       ((V : āŸØ š’Ŗ Y āŸ©) ā†’ f ā‹†āˆ™ V ļ¼ g ā‹†āˆ™ V)
                     ā†’ f ļ¼ g
to-continuous-map-ļ¼ X Y f g Ļ† =
 to-frame-homomorphism-ļ¼ (š’Ŗ Y) (š’Ŗ X) (_ā‹† f) (_ā‹† g) Ļ†
  where
   open ContinuousMapNotation X Y

\end{code}