8e6324185a
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
9 lines
203 B
Text
9 lines
203 B
Text
import standard
|
|
using tactic
|
|
|
|
theorem tst (a b : Prop) (H : a ↔ b) : b ↔ a
|
|
:= by apply iff_intro;
|
|
apply (assume Hb, iff_elim_right H Hb);
|
|
apply (assume Ha, iff_elim_left H Ha)
|
|
|
|
check tst
|