Documentation

Init.Grind.Injective

theorem Function.Injective.leftInverse {α : Sort u_1} {β : Sort u_2} (f : αβ) (hf : Injective f) [ : Nonempty α] :
(g : βα), LeftInverse g f
noncomputable def Lean.Grind.leftInv {α : Sort u} {β : Sort v} (f : αβ) (hf : Function.Injective f) [Nonempty α] :
βα
Equations
Instances For
    theorem Lean.Grind.leftInv_eq {α : Sort u} {β : Sort v} (f : αβ) (hf : Function.Injective f) [Nonempty α] (a : α) :
    f⁻¹ (f a) = a
    Equations
    • One or more equations did not get rendered due to their size.
    Instances For