Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit c057758

Browse files
ChrisHughes24johoelzl
authored andcommitted
feat(data/complex/exponential): exp_eq_one_iff
1 parent db69173 commit c057758

File tree

1 file changed

+4
-1
lines changed

1 file changed

+4
-1
lines changed

src/data/complex/exponential.lean

Lines changed: 4 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -840,6 +840,9 @@ lemma exp_injective : function.injective exp :=
840840
{ exact absurd h (ne.symm (ne_of_lt (exp_lt_exp h₁))) }
841841
end
842842

843+
@[simp] lemma exp_eq_one_iff : exp x = 1 ↔ x = 0 :=
844+
by rw ← exp_zero; exact λ h, exp_injective h, λ h, by rw [h, exp_zero]⟩
845+
843846
end real
844847

845848
namespace complex
@@ -1052,4 +1055,4 @@ by rw [exp_eq_exp_re_mul_sin_add_cos, exp_eq_exp_re_mul_sin_add_cos y,
10521055
@[simp] lemma abs_exp_of_real (x : ℝ) : abs (exp x) = real.exp x :=
10531056
by rw [← of_real_exp]; exact abs_of_nonneg (le_of_lt (real.exp_pos _))
10541057

1055-
end complex
1058+
end complex

0 commit comments

Comments
 (0)