lean2/tests/lean/refute1.lean
Leonardo de Moura 57c0006916 chore(*): cleanup lean builtin symbols, replace :: with _
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2014-01-09 08:33:52 -08:00

3 lines
94 B
Text

variables a b : Bool
axiom H : a /\ b
theorem T : a := refute (fun R, absurd (and_eliml H) R)