4946f55290
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
7 lines
225 B
Text
7 lines
225 B
Text
import logic data.unit
|
||
open bool unit decidable
|
||
|
||
constants a b c : bool
|
||
constants u v : unit
|
||
set_option pp.implicit true
|
||
check if ((a = b) ∧ (b = c) → ¬ (u = v) ∨ (a = c) → (a = c) ↔ a = tt ↔ true) then a else b
|