Add Everything files in preparation for Travis build (#36)

This commit is contained in:
Patrick Stevens
2019-08-18 12:59:13 +01:00
committed by GitHub
parent e7c54fa48a
commit 69389bb889
3 changed files with 71 additions and 0 deletions

31
Everything/WithK.agda Normal file
View File

@@ -0,0 +1,31 @@
{-# OPTIONS --warning=error --safe #-}
-- This file contains everything that is --safe, but uses K.
open import PrimeNumbers
open import Numbers.Integers
open import Numbers.Rationals
open import Numbers.RationalsLemmas
open import Numbers.BinaryNaturals.Multiplication -- TODO there's no reason for this to need K
open import Numbers.BinaryNaturals.Order -- TODO likewise this
open import Logic.PropositionalLogic
open import Logic.PropositionalLogicExamples
open import Logic.PropositionalAxiomsTautology
open import IntegersModN
open import Sets.FinSetWithK
open import Vectors
open import KeyValue
open import KeyValueWithDomain
open import Rings.Examples.Examples
open import Rings.Examples.Proofs
open import Groups.FreeGroups
open import Groups.Groups2
module Everything.WithK where