lean2/tests/lean/pattern_bug1.lean
2015-12-05 19:38:24 -08:00

3 lines
137 B
Text

constants {A : Type} (P : A → Prop) (R : A → A → Prop)
definition H [forward] : ∀ a, (: P a :) → ∃ b, R a b := sorry
print H