Skip to content

Commit 2b362e7

Browse files
gallaisplt-amy
authored andcommitted
[ re #1993 ] Simplifying the dependency graph (#1995)
1 parent bb523b0 commit 2b362e7

File tree

107 files changed

+243
-268
lines changed

Some content is hidden

Large Commits have some content hidden by default. Use the searchbox below for content that may be hidden.

107 files changed

+243
-268
lines changed

src/Algebra/Consequences/Setoid.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -15,7 +15,7 @@ open Setoid S renaming (Carrier to A)
1515
open import Algebra.Core
1616
open import Algebra.Definitions _≈_
1717
open import Data.Sum.Base using (inj₁; inj₂)
18-
open import Data.Product using (_,_)
18+
open import Data.Product.Base using (_,_)
1919
open import Function.Base using (_$_)
2020
import Function.Definitions as FunDefs
2121
import Relation.Binary.Consequences as Bin

src/Algebra/Construct/LexProduct/Base.agda

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -8,10 +8,10 @@
88

99
open import Algebra.Core using (Op₂)
1010
open import Data.Bool.Base using (true; false)
11-
open import Data.Product using (_×_; _,_)
11+
open import Data.Product.Base using (_×_; _,_)
1212
open import Relation.Binary.Core using (Rel)
1313
open import Relation.Binary.Definitions using (Decidable)
14-
open import Relation.Nullary.Decidable using (does; yes; no)
14+
open import Relation.Nullary.Decidable.Core using (does; yes; no)
1515

1616
module Algebra.Construct.LexProduct.Base
1717
{a b ℓ} {A : Set a} {B : Set b}

src/Algebra/Construct/NaturalChoice/MinMaxOp.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -11,7 +11,7 @@ open import Algebra.Core
1111
open import Algebra.Bundles
1212
open import Algebra.Construct.NaturalChoice.Base
1313
open import Data.Sum.Base as Sum using (inj₁; inj₂; [_,_])
14-
open import Data.Product using (_,_)
14+
open import Data.Product.Base using (_,_)
1515
open import Function.Base using (id; _∘_; flip)
1616
open import Relation.Binary
1717
open import Relation.Binary.Consequences

src/Algebra/Construct/NaturalChoice/MinOp.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -11,7 +11,7 @@ open import Algebra.Core
1111
open import Algebra.Bundles
1212
open import Algebra.Construct.NaturalChoice.Base
1313
open import Data.Sum.Base as Sum using (inj₁; inj₂; [_,_])
14-
open import Data.Product using (_,_)
14+
open import Data.Product.Base using (_,_)
1515
open import Function.Base using (id; _∘_)
1616
open import Relation.Binary
1717
open import Relation.Binary.Consequences

src/Algebra/Definitions.agda

Lines changed: 5 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -15,17 +15,17 @@
1515

1616
{-# OPTIONS --cubical-compatible --safe #-}
1717

18-
open import Relation.Binary.Core
19-
open import Relation.Nullary.Negation using (¬_)
18+
open import Relation.Binary.Core using (Rel; _Preserves_⟶_; _Preserves₂_⟶_⟶_)
19+
open import Relation.Nullary.Negation.Core using (¬_)
2020

2121
module Algebra.Definitions
2222
{a ℓ} {A : Set a} -- The underlying set
2323
(_≈_ : Rel A ℓ) -- The underlying equality
2424
where
2525

26-
open import Algebra.Core
27-
open import Data.Product
28-
open import Data.Sum.Base
26+
open import Algebra.Core using (Op₁; Op₂)
27+
open import Data.Product.Base using (_×_; ∃-syntax)
28+
open import Data.Sum.Base using (_⊎_)
2929

3030
------------------------------------------------------------------------
3131
-- Properties of operations

src/Algebra/Definitions/RawMagma.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -11,7 +11,7 @@
1111
{-# OPTIONS --cubical-compatible --safe #-}
1212

1313
open import Algebra.Bundles using (RawMagma)
14-
open import Data.Product using (_×_; ∃)
14+
open import Data.Product.Base using (_×_; ∃)
1515
open import Level using (_⊔_)
1616
open import Relation.Binary.Core
1717
open import Relation.Nullary.Negation using (¬_)

src/Algebra/Lattice/Properties/BooleanAlgebra.agda

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -23,9 +23,9 @@ open import Algebra.Bundles
2323
open import Algebra.Lattice.Structures _≈_
2424
open import Relation.Binary.Reasoning.Setoid setoid
2525
open import Relation.Binary
26-
open import Function.Base
26+
open import Function.Base using (id; _$_; _⟨_⟩_)
2727
open import Function.Bundles using (_⇔_; module Equivalence)
28-
open import Data.Product using (_,_)
28+
open import Data.Product.Base using (_,_)
2929

3030
------------------------------------------------------------------------
3131
-- Export properties from distributive lattices

src/Algebra/Lattice/Properties/Lattice.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -11,7 +11,7 @@ import Algebra.Lattice.Properties.Semilattice as SemilatticeProperties
1111
open import Relation.Binary
1212
import Relation.Binary.Lattice as R
1313
open import Function.Base
14-
open import Data.Product using (_,_; swap)
14+
open import Data.Product.Base using (_,_; swap)
1515

1616
module Algebra.Lattice.Properties.Lattice
1717
{l₁ l₂} (L : Lattice l₁ l₂) where

src/Algebra/Lattice/Properties/Semilattice.agda

Lines changed: 2 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -6,11 +6,8 @@
66

77
{-# OPTIONS --cubical-compatible --safe #-}
88

9-
open import Algebra.Lattice
10-
open import Algebra.Structures
11-
open import Function
12-
open import Data.Product
13-
open import Relation.Binary
9+
open import Algebra.Lattice.Bundles using (Semilattice)
10+
open import Relation.Binary.Bundles using (Poset)
1411
import Relation.Binary.Lattice as B
1512
import Relation.Binary.Properties.Poset as PosetProperties
1613

src/Algebra/Lattice/Structures.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -14,7 +14,7 @@
1414
{-# OPTIONS --cubical-compatible --safe #-}
1515

1616
open import Algebra.Core
17-
open import Data.Product using (proj₁; proj₂)
17+
open import Data.Product.Base using (proj₁; proj₂)
1818
open import Level using (_⊔_)
1919
open import Relation.Binary using (Rel; Setoid; IsEquivalence)
2020

0 commit comments

Comments
 (0)