{-# OPTIONS --safe #-}
module Cubical.Algebra.CommRing.Instances.Unit where

open import Cubical.Foundations.Prelude

open import Cubical.Data.Unit

open import Cubical.Algebra.Ring
open import Cubical.Algebra.CommRing

private
  variable
     : Level

open CommRingStr

UnitCommRing :  {}  CommRing 
fst UnitCommRing = Unit*
0r (snd UnitCommRing) = tt*
1r (snd UnitCommRing) = tt*
_+_ (snd UnitCommRing) = λ _ _  tt*
_·_ (snd UnitCommRing) = λ _ _  tt*
- snd UnitCommRing = λ _  tt*
isCommRing (snd UnitCommRing) =
  makeIsCommRing isSetUnit*  _ _ _  refl)  { tt*  refl })  _  refl)
                  _ _  refl)  _ _ _  refl)  { tt*  refl })
                  _ _ _  refl)  _ _  refl)