Zulip Chat Archive
Stream: Is there code for X?
Topic: lemma exp_pi_mul_I_half : exp (↑real.pi * I / 2) = I :=
Mark Gerads (Jul 13 2022 at 01:03):
I need to simplify this in a proof
lemma exp_pi_mul_I_half : exp (↑real.pi * I / 2) = I :=
Currently attempting proof.
Kevin Buzzard (Jul 13 2022 at 02:55):
import analysis.special_functions.trigonometric.basic
open complex
noncomputable abbreviation pi := real.pi
lemma exp_pi_mul_I_half : exp (↑pi * I / 2) = I :=
begin
-- would rather the /2 is real
rw (show (pi : ℂ) * I / 2 = (pi / 2 : ℝ) * I, by {simp, ring, } ),
-- now apply Euler, which was bound to be there in some form
rw exp_mul_I,
-- now hope simplifier knows all the facts about cos(pi/2) etc.
simp,
-- it does!
end
Last updated: Dec 20 2023 at 11:08 UTC