File tree 10 files changed +24
-22
lines changed
Function/Indexed/Relation/Binary
10 files changed +24
-22
lines changed Original file line number Diff line number Diff line change 10
10
11
11
{-# OPTIONS --cubical-compatible --safe #-}
12
12
13
- open import Algebra.Bundles using (RawMagma)
13
+ open import Algebra.Bundles.Raw using (RawMagma)
14
14
open import Data.Product.Base using (_×_; ∃)
15
15
open import Level using (_⊔_)
16
- open import Relation.Binary.Core
17
- open import Relation.Nullary.Negation using (¬_)
16
+ open import Relation.Binary.Core using (Rel)
17
+ open import Relation.Nullary.Negation.Core using (¬_)
18
18
19
19
module Algebra.Definitions.RawMagma
20
20
{a ℓ} (M : RawMagma a ℓ)
Original file line number Diff line number Diff line change @@ -21,7 +21,7 @@ module Algebra.Structures
21
21
-- The file is divided into sections depending on the arities of the
22
22
-- components of the algebraic structure.
23
23
24
- open import Algebra.Core
24
+ open import Algebra.Core using (Op₁; Op₂)
25
25
open import Algebra.Definitions _≈_
26
26
import Algebra.Consequences.Setoid as Consequences
27
27
open import Data.Product.Base using (_,_; proj₁; proj₂)
Original file line number Diff line number Diff line change @@ -18,7 +18,7 @@ open import Function.Base using (id; _∘_)
18
18
open import Level using (_⊔_)
19
19
open import Relation.Binary.Definitions as B
20
20
open import Relation.Binary.Construct.Intersection renaming (_∩_ to _∩ᵇ_)
21
- open import Relation.Binary.PropositionalEquality
21
+ open import Relation.Binary.PropositionalEquality.Core using (refl; cong₂)
22
22
open import Relation.Unary as U renaming (_∩_ to _∩ᵘ_) hiding (_⇒_)
23
23
open import Relation.Nullary.Decidable as Dec using (_×-dec_; yes; no)
24
24
Original file line number Diff line number Diff line change @@ -15,9 +15,9 @@ open import Data.Bool.Base using (Bool; true; false; not)
15
15
open import Data.Unit.Base using (⊤)
16
16
open import Data.These.Base using (These; this; that; these)
17
17
open import Data.Product.Base as Prod using (_×_; _,_)
18
- open import Function.Base
19
- open import Relation.Nullary.Reflects
20
- open import Relation.Nullary.Decidable.Core
18
+ open import Function.Base using (const; _∘_; id)
19
+ open import Relation.Nullary.Reflects using (invert)
20
+ open import Relation.Nullary.Decidable.Core using (Dec; _because_)
21
21
22
22
private
23
23
variable
Original file line number Diff line number Diff line change 8
8
9
9
module Data.Product.Properties where
10
10
11
- open import Axiom.UniquenessOfIdentityProofs
12
- open import Data.Product.Base
11
+ open import Axiom.UniquenessOfIdentityProofs using (UIP; module Decidable⇒UIP )
12
+ open import Data.Product.Base using (_,_; Σ; _×_; map; swap; ∃; ∃₂)
13
13
open import Function.Base using (_∋_; _∘_; id)
14
14
open import Function.Bundles using (_↔_; mk↔ₛ′)
15
15
open import Level using (Level)
Original file line number Diff line number Diff line change 8
8
9
9
module Function.Indexed.Relation.Binary.Equality where
10
10
11
- open import Relation.Binary using (Setoid)
11
+ open import Relation.Binary.Bundles using (Setoid)
12
12
open import Relation.Binary.Indexed.Heterogeneous using (IndexedSetoid)
13
13
14
14
-- A variant of setoid which uses the propositional equality setoid
Original file line number Diff line number Diff line change 11
11
module Relation.Binary.Bundles where
12
12
13
13
open import Function.Base using (flip)
14
- open import Level
15
- open import Relation.Nullary.Negation using (¬_)
16
- open import Relation.Binary.Core
17
- open import Relation.Binary.Definitions
18
- open import Relation.Binary.Structures
14
+ open import Level using (Level; suc; _⊔_)
15
+ open import Relation.Nullary.Negation.Core using (¬_)
16
+ open import Relation.Binary.Core using (Rel)
17
+ open import Relation.Binary.Structures -- most of it
19
18
20
19
------------------------------------------------------------------------
21
20
-- Setoids
Original file line number Diff line number Diff line change 8
8
9
9
module Relation.Binary.PropositionalEquality.Algebra where
10
10
11
- open import Algebra
12
- open import Level
13
- open import Relation.Binary.PropositionalEquality.Core
14
- open import Relation.Binary.PropositionalEquality.Properties
11
+ open import Algebra.Bundles using (Magma)
12
+ open import Algebra.Core using (Op₂)
13
+ open import Algebra.Structures using (IsMagma)
14
+ open import Level using (Level)
15
+ open import Relation.Binary.PropositionalEquality.Core using (_≡_; cong₂)
16
+ open import Relation.Binary.PropositionalEquality.Properties using (isEquivalence)
15
17
16
18
private
17
19
variable
Original file line number Diff line number Diff line change 21
21
{-# OPTIONS --cubical-compatible --safe #-}
22
22
23
23
open import Relation.Binary.Bundles using (Setoid)
24
- open import Relation.Binary.Reasoning.Syntax
24
+ open import Relation.Binary.Reasoning.Syntax using ( module ≈-syntax )
25
25
26
26
module Relation.Binary.Reasoning.Setoid {s₁ s₂} (S : Setoid s₁ s₂) where
27
27
Original file line number Diff line number Diff line change 9
9
open import Level using (Level; _⊔_; suc)
10
10
open import Relation.Nullary.Decidable.Core
11
11
using (Dec; True; toWitness)
12
- open import Relation.Nullary.Negation using (contradiction)
12
+ open import Relation.Nullary.Negation.Core using (contradiction)
13
13
open import Relation.Binary.Core using (Rel; REL; _⇒_)
14
14
open import Relation.Binary.Definitions
15
+ using (_Respectsʳ_; Asymmetric; Trans; Sym; Reflexive)
15
16
open import Relation.Binary.PropositionalEquality.Core as ≡
16
17
using (_≡_)
17
18
You can’t perform that action at this time.
0 commit comments