Skip to content

Commit

Permalink
docs(algebra/hom/group, tactic/push_neg): add docs to resolve some li…
Browse files Browse the repository at this point in the history
…nt errors (#17225)
  • Loading branch information
adomani committed Oct 30, 2022
1 parent 7f5bf38 commit da8ded3
Show file tree
Hide file tree
Showing 2 changed files with 8 additions and 6 deletions.
7 changes: 4 additions & 3 deletions src/algebra/hom/group.lean
Expand Up @@ -594,11 +594,11 @@ fun_like.coe_injective h
lemma one_hom.ext_iff [has_one M] [has_one N] {f g : one_hom M N} : f = g ↔ ∀ x, f x = g x :=
fun_like.ext_iff
/-- Deprecated: use `fun_like.ext_iff` instead. -/
@[to_additive]
@[to_additive "Deprecated: use `fun_like.ext_iff` instead."]
lemma mul_hom.ext_iff [has_mul M] [has_mul N] {f g : M →ₙ* N} : f = g ↔ ∀ x, f x = g x :=
fun_like.ext_iff
/-- Deprecated: use `fun_like.ext_iff` instead. -/
@[to_additive]
@[to_additive "Deprecated: use `fun_like.ext_iff` instead."]
lemma monoid_hom.ext_iff [mul_one_class M] [mul_one_class N]
{f g : M →* N} : f = g ↔ ∀ x, f x = g x :=
fun_like.ext_iff
Expand Down Expand Up @@ -806,7 +806,8 @@ lemma monoid_with_zero_hom.comp_apply [mul_zero_one_class M] [mul_zero_one_class
g.comp f x = g (f x) := rfl

/-- Composition of monoid homomorphisms is associative. -/
@[to_additive] lemma one_hom.comp_assoc {Q : Type*} [has_one M] [has_one N] [has_one P] [has_one Q]
@[to_additive "Composition of additive monoid homomorphisms is associative."]
lemma one_hom.comp_assoc {Q : Type*} [has_one M] [has_one N] [has_one P] [has_one Q]
(f : one_hom M N) (g : one_hom N P) (h : one_hom P Q) :
(h.comp g).comp f = h.comp (g.comp f) := rfl
@[to_additive] lemma mul_hom.comp_assoc {Q : Type*} [has_mul M] [has_mul N] [has_mul P] [has_mul Q]
Expand Down
7 changes: 4 additions & 3 deletions src/tactic/push_neg.lean
Expand Up @@ -2,13 +2,14 @@
Copyright (c) 2019 Patrick Massot All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Patrick Massot, Simon Hudon
A tactic pushing negations into an expression
-/

import tactic.core
import logic.basic

/-!
# A tactic pushing negations into an expression
-/

open tactic expr

/- Enable the option `trace.push_neg.use_distrib` in order to have `¬ (p ∧ q)` normalized to
Expand Down

0 comments on commit da8ded3

Please sign in to comment.