Skip to content

Commit

Permalink
revert: remove spurious imports
Browse files Browse the repository at this point in the history
  • Loading branch information
jamesmckinna committed Dec 9, 2024
1 parent 5e7cd5c commit ad4b103
Showing 1 changed file with 0 additions and 1 deletion.
Original file line number Diff line number Diff line change
Expand Up @@ -10,7 +10,6 @@ module Data.List.Relation.Binary.Sublist.Propositional.Properties
{a} {A : Set a} where

open import Data.List.Base using (List; []; _∷_; map)
open import Data.List.Properties using (map-id)
open import Data.List.Membership.Propositional using (_∈_)
open import Data.List.Relation.Unary.All using (All; []; _∷_)
open import Data.List.Relation.Unary.Any using (Any; here; there)
Expand Down

0 comments on commit ad4b103

Please sign in to comment.