-
Notifications
You must be signed in to change notification settings - Fork 246
/
Copy pathHeytingCommutativeRing.agda
39 lines (29 loc) · 1.29 KB
/
HeytingCommutativeRing.agda
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
30
31
32
33
34
35
36
37
38
39
------------------------------------------------------------------------
-- The Agda standard library
--
-- Properties of Heyting Commutative Rings
------------------------------------------------------------------------
{-# OPTIONS --cubical-compatible --safe #-}
open import Algebra.Apartness.Bundles using (HeytingCommutativeRing)
module Algebra.Apartness.Properties.HeytingCommutativeRing
{c ℓ₁ ℓ₂} (HCR : HeytingCommutativeRing c ℓ₁ ℓ₂) where
open import Algebra.Bundles using (CommutativeRing)
open HeytingCommutativeRing HCR using (commutativeRing)
open CommutativeRing commutativeRing using (ring)
open import Algebra.Properties.Ring ring using (x-0#≈x)
------------------------------------------------------------------------
-- DEPRECATED NAMES
------------------------------------------------------------------------
-- Please use the new names as continuing support for the old names is
-- not guaranteed.
-- Version 2.3
x-0≈x = x-0#≈x
{-# WARNING_ON_USAGE x-0≈x
"Warning: x-0≈x was deprecated in v2.3.
Please use Algebra.Properties.Ring.x-0#≈x instead."
#-}
open HeytingCommutativeRing HCR public using (#-sym)
{-# WARNING_ON_USAGE #-sym
"Warning: #-sym was deprecated in v2.3.
Please use Algebra.Apartness.Structures.IsHeytingCommutativeRing.#-sym instead."
#-}