Skip to content

Commit

Permalink
fix(library/init/function): make injective semireducible (#604)
Browse files Browse the repository at this point in the history
  • Loading branch information
fpvandoorn committed Aug 18, 2021
1 parent fe0061d commit 03a6a60
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion library/init/function.lean
Expand Up @@ -70,7 +70,7 @@ lemma comp.assoc (f : φ → δ) (g : β → φ) (h : α → β) : (f ∘ g) ∘
lemma comp_const_right (f : β → φ) (b : β) : f ∘ (const α b) = const α (f b) := rfl

/-- A function `f : α → β` is called injective if `f x = f y` implies `x = y`. -/
@[reducible] def injective (f : α → β) : Prop := ∀ ⦃a₁ a₂⦄, f a₁ = f a₂ → a₁ = a₂
def injective (f : α → β) : Prop := ∀ ⦃a₁ a₂⦄, f a₁ = f a₂ → a₁ = a₂

lemma injective.comp {g : β → φ} {f : α → β} (hg : injective g) (hf : injective f) :
injective (g ∘ f) :=
Expand Down

0 comments on commit 03a6a60

Please sign in to comment.