File tree 2 files changed +2
-2
lines changed
2 files changed +2
-2
lines changed Original file line number Diff line number Diff line change @@ -13,7 +13,7 @@ open import Relation.Binary.Core using (Rel)
13
13
open import Relation.Binary.Bundles using (ApartnessRelation)
14
14
open import Algebra.Core using (Op₁; Op₂)
15
15
open import Algebra.Bundles using (CommutativeRing)
16
- open import Algebra.Apartness.Structures
16
+ open import Algebra.Apartness.Structures using (IsHeytingCommutativeRing; IsHeytingField)
17
17
18
18
record HeytingCommutativeRing c ℓ₁ ℓ₂ : Set (suc (c ⊔ ℓ₁ ⊔ ℓ₂)) where
19
19
infix 8 -_
Original file line number Diff line number Diff line change @@ -14,9 +14,9 @@ open import Algebra.Core using (Op₂)
14
14
open import Algebra.Definitions
15
15
using (Congruent₂; Associative; LeftIdentity; RightIdentity; Identity)
16
16
open import Algebra.Structures using (IsMagma; IsSemigroup; IsMonoid)
17
- open import Relation.Binary.Construct.Add.Point.Equality renaming (_≈∙_ to lift≈)
18
17
open import Data.Product.Base using (_,_)
19
18
open import Level using (Level; _⊔_)
19
+ open import Relation.Binary.Construct.Add.Point.Equality renaming (_≈∙_ to lift≈)
20
20
open import Relation.Binary.Core using (Rel)
21
21
open import Relation.Binary.Definitions using (Reflexive)
22
22
open import Relation.Binary.Structures using (IsEquivalence)
You can’t perform that action at this time.
0 commit comments