symmetries/Cubical/Structures/Set/CMon/SList/Sort.agda

9 lines
355 B
Plaintext

{-# OPTIONS --cubical --safe --exact-split #-}
module Cubical.Structures.Set.CMon.SList.Sort where
open import Cubical.Structures.Set.CMon.SList.Sort.Base public
open import Cubical.Structures.Set.CMon.SList.Sort.Order public
open import Cubical.Structures.Set.CMon.SList.Sort.Sort public
open import Cubical.Structures.Set.CMon.SList.Sort.Equiv public