symmetries/Cubical/Structures/Set/CMon/Bag.agda

9 lines
266 B
Plaintext

{-# OPTIONS --cubical --safe --exact-split #-}
module Cubical.Structures.Set.CMon.Bag where
open import Cubical.Structures.Set.CMon.Bag.Base public
open import Cubical.Structures.Set.CMon.Bag.Free public
open import Cubical.Structures.Set.CMon.Bag.ToCList public