mirror of
https://github.com/Smaug123/agdaproofs
synced 2025-10-12 07:08:40 +00:00
32 lines
800 B
Agda
32 lines
800 B
Agda
{-# 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
|