Add Everything (#34)

This commit is contained in:
Patrick Stevens
2019-08-18 10:35:15 +01:00
committed by GitHub
parent a31ae0d1ea
commit e7c54fa48a
45 changed files with 415 additions and 378 deletions

View File

@@ -1,15 +1,16 @@
{-# OPTIONS --safe --warning=error #-}
open import LogicalFormulae
open import Setoids
open import Setoids.Setoids
open import Functions
open import Agda.Primitive using (Level; lzero; lsuc; _⊔_)
open import Naturals
open import Integers
open import FinSet
open import Groups
open import Numbers.Naturals
open import Numbers.Integers
open import Sets.FinSet
open import Groups.Groups
open import Groups.GroupDefinition
module CyclicGroups where
module Groups.CyclicGroups where
positiveEltPower : {m n : _} {A : Set m} {S : Setoid {m} {n} A} {_·_ : A A A} (G : Group S _·_) (x : A) (i : ) A
positiveEltPower G x 0 = Group.identity G