lean2/tests/lean/run/decidable.lean

8 lines
235 B
Text
Raw Normal View History

import standard unit decidable if
using bit unit decidable
variables a b c : bit
variables u v : unit
set_option pp.implicit true
check if ((a = b) ∧ (b = c) → ¬ (u = v) (a = c) → (a = c) ↔ a = '1 ↔ true) then a else b