c9-core/plugins/node_modules/ace/demo/kitchen-sink/docs/lean.lean

10 wiersze
213 B
Plaintext

import logic
section
variables (A : Type) (p q : A → Prop)
example : (∀x : A, p x ∧ q x) → ∀y : A, p y :=
assume H : ∀x : A, p x ∧ q x,
take y : A,
show p y, from and.elim_left (H y)
end