Total order on the rationals (#17)

This commit is contained in:
Patrick Stevens
2019-01-13 12:05:30 +00:00
committed by GitHub
parent 9e22ba78f5
commit 2866b11be6
9 changed files with 624 additions and 52 deletions

View File

@@ -6,6 +6,7 @@ open import Functions
open import Agda.Primitive using (Level; lzero; lsuc; _⊔_)
open import Numbers.Naturals
open import Groups.Groups
open import Groups.GroupDefinition
module Groups.GroupsLemmas where
invInv : {a b : _} {A : Set a} {_·_ : A A A} {S : Setoid {a} {b} A} (G : Group S _·_) {x : A} Setoid.__ S (Group.inverse G (Group.inverse G x)) x