3 lines
94 B
Text
3 lines
94 B
Text
variables a b : Bool
|
|
axiom H : a /\ b
|
|
theorem T : a := refute (fun R, absurd (and_eliml H) R)
|