2023-09-23 17:12:12 -07:00
|
|
|
|
open import Lattice
|
|
|
|
|
open import Relation.Binary.PropositionalEquality as Eq using (_≡_; refl; sym; trans; cong; subst)
|
|
|
|
|
open import Relation.Binary.Definitions using (Decidable)
|
|
|
|
|
open import Agda.Primitive using (Level) renaming (_⊔_ to _⊔ℓ_)
|
|
|
|
|
|
|
|
|
|
module Lattice.MapSet {a : Level} (A : Set a) (≡-dec-A : Decidable (_≡_ {a} {A})) where
|
|
|
|
|
|
|
|
|
|
open import Lattice.Unit using (⊤) renaming (_≈_ to _≈₂_; _⊔_ to _⊔₂_; _⊓_ to _⊓₂_; isLattice to ⊤-isLattice)
|
|
|
|
|
import Lattice.Map
|
|
|
|
|
|
|
|
|
|
private module UnitMap = Lattice.Map A ⊤ _≈₂_ _⊔₂_ _⊓₂_ ≡-dec-A ⊤-isLattice
|
|
|
|
|
open UnitMap using (Map)
|
|
|
|
|
open UnitMap using
|
|
|
|
|
( _⊆_; _≈_; ≈-equiv; _⊔_; _⊓_
|
2024-02-11 21:14:49 -08:00
|
|
|
|
; isUnionSemilattice; isIntersectSemilattice; isLattice; lattice
|
2023-09-23 17:12:12 -07:00
|
|
|
|
) public
|
|
|
|
|
|
|
|
|
|
MapSet : Set a
|
|
|
|
|
MapSet = Map
|