Skip to content

Commit af28176

Browse files
authored
[imports] Data.List.Effectful.* .. Relation.Nullary (#2624)
* Imports Cleaning Data 4 * fix * fix
1 parent 098b4cf commit af28176

File tree

15 files changed

+71
-62
lines changed

15 files changed

+71
-62
lines changed

src/Data/List/Effectful/Foldable.agda

+1-1
Original file line numberDiff line numberDiff line change
@@ -15,7 +15,7 @@ open import Data.List.Base as List using (List; []; _∷_; _++_)
1515
open import Effect.Foldable using (RawFoldableWithDefaults; RawFoldable)
1616
open import Function.Base using (_∘_; id)
1717
open import Level using (Level)
18-
import Relation.Binary.PropositionalEquality.Core as ≡
18+
import Relation.Binary.PropositionalEquality.Core as ≡ using (_≡_; cong)
1919

2020
private
2121
variable

src/Data/List/Effectful/Transformer.agda

+5-6
Original file line numberDiff line numberDiff line change
@@ -9,13 +9,12 @@
99
module Data.List.Effectful.Transformer where
1010

1111
open import Data.List.Base as List using (List; []; _∷_)
12-
open import Effect.Functor
13-
open import Effect.Applicative
14-
open import Effect.Monad
15-
open import Function.Base
16-
open import Level
17-
1812
import Data.List.Effectful as List
13+
open import Effect.Functor using (RawFunctor)
14+
open import Effect.Applicative using (RawApplicative)
15+
open import Effect.Monad using (RawMonad; RawMonadT)
16+
open import Function.Base using (_∘′_; _∘_; _$_)
17+
open import Level using (Level)
1918

2019
private
2120
variable

src/Data/List/Extrema/Core.agda

+7-4
Original file line numberDiff line numberDiff line change
@@ -6,22 +6,25 @@
66

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

9-
open import Relation.Binary.Definitions using (Trans)
109
open import Relation.Binary.Bundles using (TotalOrder; Setoid)
1110

1211
module Data.List.Extrema.Core
1312
{b ℓ₁ ℓ₂} (totalOrder : TotalOrder b ℓ₁ ℓ₂) where
1413

15-
open import Algebra.Core
16-
open import Algebra.Definitions
14+
open import Algebra.Construct.LiftedChoice
15+
using (Lift; sel-≡; preservesᵒ; preservesᵇ ; forcesᵇ)
16+
open import Algebra.Core using (Op₂)
17+
open import Algebra.Definitions using (Selective)
1718
import Algebra.Construct.NaturalChoice.Min as Min
19+
using (_⊓_; x⊓y≈y⇒y≤x; x⊓y≈x⇒x≤y; ⊓-sel; ⊓-isSelectiveMagma)
1820
import Algebra.Construct.NaturalChoice.Max as Max
21+
using (_⊔_; x⊔y≈y⇒x≤y; x⊔y≈x⇒y≤x; ⊔-sel; ⊔-isSelectiveMagma)
1922
open import Data.Product.Base using (_×_; _,_)
2023
open import Data.Sum.Base using (_⊎_; inj₁; inj₂)
2124
open import Level using (Level)
2225
open import Relation.Binary.PropositionalEquality.Core using (_≡_)
26+
open import Relation.Binary.Definitions using (Trans)
2327

24-
open import Algebra.Construct.LiftedChoice
2528

2629
open TotalOrder totalOrder renaming (Carrier to B)
2730
open import Relation.Binary.Construct.NonStrictToStrict _≈_ _≤_

src/Data/List/Fresh.agda

+1-1
Original file line numberDiff line numberDiff line change
@@ -26,7 +26,7 @@ open import Relation.Nullary using (does)
2626
open import Relation.Unary as U using (Pred)
2727
open import Relation.Binary.Core using (Rel)
2828
import Relation.Binary.Definitions as B
29-
open import Relation.Nary
29+
open import Relation.Nary using (∀[_]; _⇒_)
3030

3131
private
3232
variable

src/Data/List/Fresh/Membership/Setoid.agda

+3-3
Original file line numberDiff line numberDiff line change
@@ -6,15 +6,15 @@
66

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

9-
open import Relation.Binary.Core using (Rel)
109
open import Relation.Binary.Bundles using (Setoid)
1110

1211
module Data.List.Fresh.Membership.Setoid {c ℓ} (S : Setoid c ℓ) where
1312

1413
open import Level using (Level; _⊔_)
15-
open import Data.List.Fresh
14+
open import Data.List.Fresh using (List#)
1615
open import Data.List.Fresh.Relation.Unary.Any as Any using (Any)
17-
open import Relation.Nullary
16+
open import Relation.Binary.Core using (Rel)
17+
open import Relation.Nullary.Negation.Core using (¬_)
1818

1919
open Setoid S renaming (Carrier to A)
2020

src/Data/List/Fresh/Membership/Setoid/Properties.agda

+17-15
Original file line numberDiff line numberDiff line change
@@ -6,30 +6,32 @@
66

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

9-
open import Relation.Binary.Core using (Rel)
109
open import Relation.Binary.Bundles using (Setoid)
1110

12-
module Data.List.Fresh.Membership.Setoid.Properties {c ℓ} (S : Setoid c ℓ) where
11+
module Data.List.Fresh.Membership.Setoid.Properties {c ℓ} (S : Setoid c ℓ)
12+
where
1313

1414
open import Level using (Level; _⊔_)
15-
open import Data.Empty
16-
open import Data.Nat.Base
17-
open import Data.Nat.Properties
15+
open import Data.List.Fresh
16+
open import Data.List.Fresh.Properties using (fresh-respectsˡ)
17+
open import Data.List.Fresh.Membership.Setoid S using (_∈_; _∉_)
18+
open import Data.List.Fresh.Relation.Unary.Any using (Any; here; there; _─_)
19+
import Data.List.Fresh.Relation.Unary.Any.Properties as List#
20+
using (length-remove)
21+
open import Data.Empty using (⊥; ⊥-elim)
22+
open import Data.Nat.Base using (ℕ; suc; zero; _≤_; _<_; z≤n; s≤s; z<s; s<s)
23+
open import Data.Nat.Properties using (module ≤-Reasoning)
1824
open import Data.Product.Base using (∃; _×_; _,_)
1925
open import Data.Sum.Base as Sum using (_⊎_; inj₁; inj₂; fromInj₂)
20-
2126
open import Function.Base using (id; _∘′_; _$_)
22-
open import Relation.Nullary
27+
open import Relation.Binary.Core using (Rel)
28+
open import Relation.Nullary.Negation.Core using (¬_)
29+
open import Relation.Nullary using (Irrelevant)
2330
open import Relation.Unary as Unary using (Pred)
24-
import Relation.Binary.Definitions as Binary
31+
import Relation.Binary.Definitions as Binary using (_Respectsˡ_; Irrelevant)
2532
import Relation.Binary.PropositionalEquality.Core as ≡
26-
open import Relation.Nary
27-
28-
open import Data.List.Fresh
29-
open import Data.List.Fresh.Properties
30-
open import Data.List.Fresh.Membership.Setoid S
31-
open import Data.List.Fresh.Relation.Unary.Any using (Any; here; there; _─_)
32-
import Data.List.Fresh.Relation.Unary.Any.Properties as List#
33+
using (_≡_; cong; sym; subst)
34+
open import Relation.Nary using (∀[_]; _⇒_)
3335

3436
open Setoid S renaming (Carrier to A)
3537

src/Data/List/Fresh/NonEmpty.agda

+1-1
Original file line numberDiff line numberDiff line change
@@ -8,11 +8,11 @@
88

99
module Data.List.Fresh.NonEmpty where
1010

11-
open import Level using (Level; _⊔_)
1211
open import Data.List.Fresh as List# using (List#; []; cons; fresh)
1312
open import Data.Maybe.Base using (Maybe; nothing; just)
1413
open import Data.Nat.Base using (ℕ; suc)
1514
open import Data.Product.Base using (_×_; _,_)
15+
open import Level using (Level; _⊔_)
1616
open import Relation.Binary.Core using (Rel)
1717

1818
private

src/Data/List/Fresh/Properties.agda

+5-4
Original file line numberDiff line numberDiff line change
@@ -8,14 +8,15 @@
88

99
module Data.List.Fresh.Properties where
1010

11-
open import Level using (Level; _⊔_)
11+
open import Data.List.Fresh using (List#; _∷#_; _#_; Empty; NonEmpty; cons; [])
1212
open import Data.Product.Base using (_,_)
13-
open import Relation.Nullary
13+
open import Level using (Level; _⊔_)
14+
open import Relation.Nullary.Decidable using (Dec; yes; no)
15+
open import Relation.Nullary.Negation using (¬_)
1416
open import Relation.Unary as U using (Pred)
15-
import Relation.Binary.Definitions as B
17+
import Relation.Binary.Definitions as B using (_Respectsˡ_; Irrelevant)
1618
open import Relation.Binary.Core using (Rel)
1719

18-
open import Data.List.Fresh
1920

2021
private
2122
variable

src/Data/List/Fresh/Relation/Unary/All.agda

+5-4
Original file line numberDiff line numberDiff line change
@@ -8,16 +8,17 @@
88

99
module Data.List.Fresh.Relation.Unary.All where
1010

11-
open import Level using (Level; _⊔_; Lift)
11+
open import Data.List.Fresh using (List#; []; cons; _∷#_; _#_)
12+
open import Data.List.Fresh.Relation.Unary.Any as Any using (Any; here; there)
1213
open import Data.Product.Base using (_×_; _,_; proj₁; uncurry)
1314
open import Data.Sum.Base as Sum using (inj₁; inj₂; [_,_]′)
1415
open import Function.Base using (_∘_; _$_)
16+
open import Level using (Level; _⊔_; Lift)
1517
open import Relation.Nullary.Decidable as Dec using (Dec; yes; no; _×-dec_)
16-
open import Relation.Unary as U
18+
open import Relation.Unary as U
19+
using (Pred; IUniversal; Universal; Decidable; _⇒_; _∪_; _∩_)
1720
open import Relation.Binary.Core using (Rel)
1821

19-
open import Data.List.Fresh using (List#; []; cons; _∷#_; _#_)
20-
open import Data.List.Fresh.Relation.Unary.Any as Any using (Any; here; there)
2122

2223
private
2324
variable

src/Data/List/Fresh/Relation/Unary/All/Properties.agda

+7-6
Original file line numberDiff line numberDiff line change
@@ -8,18 +8,19 @@
88

99
module Data.List.Fresh.Relation.Unary.All.Properties where
1010

11-
open import Level using (Level; _⊔_; Lift)
12-
open import Data.Empty
11+
open import Data.List.Fresh using (List#; []; cons; _∷#_; _#_)
12+
open import Data.List.Fresh.Relation.Unary.All using (All; []; _∷_; append)
13+
open import Data.Empty using (⊥; ⊥-elim)
1314
open import Data.Nat.Base using (ℕ; zero; suc)
1415
open import Data.Product.Base using (_,_)
1516
open import Function.Base using (_∘′_)
16-
open import Relation.Nullary
17-
open import Relation.Unary as U
17+
open import Level using (Level; _⊔_; Lift)
18+
open import Relation.Nullary.Negation.Core using (¬_)
19+
open import Relation.Unary as U using (Pred)
1820
open import Relation.Binary.Core using (Rel)
1921
open import Relation.Binary.PropositionalEquality.Core using (_≡_; refl; cong)
2022

21-
open import Data.List.Fresh using (List#; []; cons; _∷#_; _#_)
22-
open import Data.List.Fresh.Relation.Unary.All
23+
2324

2425
private
2526
variable

src/Data/List/Fresh/Relation/Unary/Any.agda

+3-3
Original file line numberDiff line numberDiff line change
@@ -9,16 +9,16 @@
99
module Data.List.Fresh.Relation.Unary.Any where
1010

1111
open import Level using (Level; _⊔_; Lift)
12+
open import Data.List.Fresh using (List#; []; cons; _∷#_; _#_)
1213
open import Data.Product.Base using (∃; _,_; -,_)
1314
open import Data.Sum.Base using (_⊎_; [_,_]′; inj₁; inj₂)
1415
open import Function.Bundles using (_⇔_; mk⇔)
16+
open import Level using (Level; _⊔_; Lift)
1517
open import Relation.Nullary.Negation using (¬_; contradiction)
1618
open import Relation.Nullary.Decidable as Dec using (Dec; no; _⊎-dec_)
17-
open import Relation.Unary as U
19+
open import Relation.Unary as U using (Pred; IUniversal; Universal; Decidable; _⇒_; _∪_; _∩_)
1820
open import Relation.Binary.Core using (Rel)
1921

20-
open import Data.List.Fresh using (List#; []; cons; _∷#_; _#_)
21-
2222
private
2323
variable
2424
a p q r : Level

src/Data/List/Fresh/Relation/Unary/Any/Properties.agda

+8-8
Original file line numberDiff line numberDiff line change
@@ -8,24 +8,24 @@
88

99
module Data.List.Fresh.Relation.Unary.Any.Properties where
1010

11-
open import Level using (Level; _⊔_; Lift)
1211
open import Data.Bool.Base using (true; false)
13-
open import Data.Empty
12+
open import Data.Empty using (⊥; ⊥-elim)
13+
open import Data.List.Fresh using (List#; _∷#_; _#_; NonEmpty; cons; length; [])
14+
open import Data.List.Fresh.Relation.Unary.All using (All; _∷_; append; [])
15+
open import Data.List.Fresh.Relation.Unary.Any using (Any; here; there; _─_)
1416
open import Data.Nat.Base using (ℕ; zero; suc)
1517
open import Data.Product.Base using (_,_)
1618
open import Data.Sum.Base as Sum using (_⊎_; inj₁; inj₂)
1719
open import Function.Base using (_∘′_)
20+
open import Level using (Level; _⊔_; Lift)
1821
open import Relation.Nullary.Reflects using (invert)
19-
open import Relation.Nullary
22+
open import Relation.Nullary.Negation.Core using (¬_)
23+
open import Relation.Nullary.Decidable.Core
2024
open import Relation.Unary as U using (Pred)
2125
open import Relation.Binary.Core using (Rel)
22-
open import Relation.Nary
26+
open import Relation.Nary using (∀[_]; _⇒_; ∁; Decidable)
2327
open import Relation.Binary.PropositionalEquality.Core using (_≡_; refl; cong)
2428

25-
open import Data.List.Fresh
26-
open import Data.List.Fresh.Relation.Unary.All
27-
open import Data.List.Fresh.Relation.Unary.Any
28-
2929
private
3030
variable
3131
a b p q r s : Level

src/Data/List/Kleene/AsList.agda

+1-1
Original file line numberDiff line numberDiff line change
@@ -18,7 +18,7 @@ private
1818
B : Set b
1919
C : Set c
2020

21-
import Data.List.Kleene.Base as Kleene
21+
import Data.List.Kleene.Base as Kleene using ([])
2222

2323
------------------------------------------------------------------------
2424
-- Here we import half of the functions from Data.KleeneList: the half

src/Data/List/Kleene/Base.agda

+2-2
Original file line numberDiff line numberDiff line change
@@ -8,15 +8,15 @@
88

99
module Data.List.Kleene.Base where
1010

11+
open import Algebra.Core using (Op₂)
1112
open import Data.Product.Base as Product
1213
using (_×_; _,_; map₂; map₁; proj₁; proj₂)
1314
open import Data.Nat.Base as ℕ using (ℕ; suc; zero)
1415
open import Data.Maybe.Base as Maybe using (Maybe; just; nothing; maybe′)
1516
open import Data.Sum.Base as Sum using (_⊎_; inj₁; inj₂)
17+
open import Function.Base using (id; _$_; _∘_)
1618
open import Level using (Level)
1719

18-
open import Algebra.Core using (Op₂)
19-
open import Function.Base
2020

2121
private
2222
variable

src/Relation/Nary.agda

+5-3
Original file line numberDiff line numberDiff line change
@@ -15,18 +15,20 @@ module Relation.Nary where
1515
------------------------------------------------------------------------
1616

1717
open import Level using (Level; _⊔_; Lift)
18-
open import Data.Unit.Base
18+
open import Data.Unit.Base using (⊤)
1919
open import Data.Bool.Base using (true; false)
20-
open import Data.Empty
20+
open import Data.Empty using (⊥; ⊥-elim)
2121
open import Data.Nat.Base using (zero; suc)
2222
open import Data.Product.Base as Product using (_×_; _,_)
2323
open import Data.Product.Nary.NonDependent
2424
open import Data.Sum.Base using (_⊎_)
2525
open import Function.Base using (_$_; _∘′_)
2626
open import Function.Nary.NonDependent
2727
open import Relation.Nullary.Negation using (¬_)
28-
open import Relation.Nullary.Decidable as Dec using (Dec; yes; no; _because_; _×-dec_)
28+
open import Relation.Nullary.Decidable.Core as Dec
29+
using (Dec; yes; no; _because_; _×-dec_)
2930
import Relation.Unary as Unary
31+
using (Pred; Satisfiable; Universal; IUniversal)
3032
open import Relation.Binary.PropositionalEquality.Core using (_≡_; cong; subst)
3133

3234
private

0 commit comments

Comments
 (0)