Move Functions (#119)

This commit is contained in:
Patrick Stevens
2020-04-18 17:47:27 +01:00
committed by GitHub
parent 84a146f72c
commit 1831ef49c4
112 changed files with 203 additions and 193 deletions

View File

@@ -1,6 +1,6 @@
{-# OPTIONS --warning=error --safe --without-K #-}
open import Functions
open import Functions.Definition
open import Groups.Definition
open import Groups.Homomorphisms.Definition
open import Setoids.Setoids
@@ -25,7 +25,6 @@ quotientGroupLemma' {S = S} {T = T} G {H = H} f fx=fy = transferToRight H (trans
open Setoid T
open Equivalence eq
projectionMapIsGroupHom : GroupHom G (quotientGroupByHom G fHom) id
GroupHom.groupHom projectionMapIsGroupHom {x} {y} = quotientGroupLemma G fHom (Equivalence.reflexive (Setoid.eq T))
GroupHom.wellDefined projectionMapIsGroupHom x=y = quotientGroupLemma G fHom (GroupHom.wellDefined fHom x=y)