mirror of
https://github.com/Smaug123/agdaproofs
synced 2025-10-12 23:28:39 +00:00
Total order on the rationals (#17)
This commit is contained in:
@@ -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
|
||||
|
Reference in New Issue
Block a user