Skip to content

Commit

Permalink
fix(group_theory/quotient_group): remove duplicate group_hom instance
Browse files Browse the repository at this point in the history
  • Loading branch information
ChrisHughes24 committed Feb 11, 2019
1 parent 4b84aac commit eb9d710
Showing 1 changed file with 0 additions and 5 deletions.
5 changes: 0 additions & 5 deletions src/group_theory/quotient_group.lean
Expand Up @@ -79,11 +79,6 @@ attribute [to_additive quotient_add_group.coe_neg] coe_inv

local notation ` Q ` := quotient N

instance is_group_hom_quotient_group_mk : is_group_hom (mk : G → Q) :=
by refine {..}; intros; refl
attribute [to_additive quotient_add_group.is_add_group_hom_quotient_add_group_mk] quotient_group.is_group_hom_quotient_group_mk
attribute [to_additive quotient_add_group.is_add_group_hom_quotient_add_group_mk.equations._eqn_1] quotient_group.is_group_hom_quotient_group_mk.equations._eqn_1

def lift (φ : G → H) [is_group_hom φ] (HN : ∀x∈N, φ x = 1) (q : Q) : H :=
q.lift_on' φ $ assume a b (hab : a⁻¹ * b ∈ N),
(calc φ a = φ a * 1 : by simp
Expand Down

0 comments on commit eb9d710

Please sign in to comment.