lean2/tests/lean/run/decidable.lean

12 lines
250 B
Text
Raw Normal View History

import standard unit decidable
using bit unit decidable
variables a b c : bit
variables u v : unit
theorem tst : decidable ((a = b) ∧ (b = c) → ¬ (u = v) (a = c) → (a = c) ↔ a = '1 ↔ true)
(*
print(get_env():find("tst"):value())
*)