-- This is the preferred version of the integers in the library. Other
-- versions can be found in the MoreInts directory.
{-# OPTIONS --safe #-}
module Cubical.Data.Int where

open import Cubical.Data.Int.Base public
open import Cubical.Data.Int.Properties public