lean2/tests/lean/run/blast_simp2.lean

4 lines
83 B
Text

definition tst1 (a b : Prop) : a ∧ b ∧ true → b ∧ a :=
by simp
print tst1