~ubuntu-branches/ubuntu/utopic/agda-stdlib/utopic-proposed

« back to all changes in this revision

Viewing changes to src/Data/Fin/Subset.agda

  • Committer: Package Import Robot
  • Author(s): Iain Lane
  • Date: 2014-08-05 09:46:46 UTC
  • mfrom: (1.1.6)
  • Revision ID: package-import@ubuntu.com-20140805094646-zqd0c4m8ndngqg6x
Tags: 0.8-1
* [4ca6fd0] Update debian/watch to fetch tarballs from github
* [84d4313] Imported Upstream version 0.8
* [7b08243] debian/control: Require agda 2.4.x per upstream
* [37e7e10] debian/control: Standards-Version → 3.9.5, no changes required.
* [9051b9d] Run upstream's "GenerateEverything" script

Show diffs side-by-side

added added

removed removed

Lines of Context:
7
7
module Data.Fin.Subset where
8
8
 
9
9
open import Algebra
10
 
import Algebra.Props.BooleanAlgebra as BoolAlgProp
11
 
import Algebra.Props.BooleanAlgebra.Expression as BAExpr
 
10
import Algebra.Properties.BooleanAlgebra as BoolAlgProp
 
11
import Algebra.Properties.BooleanAlgebra.Expression as BAExpr
12
12
import Data.Bool.Properties as BoolProp
13
13
open import Data.Fin
14
14
open import Data.List as List using (List)