lean2/tests/lean/pattern_bug1.lean

4 lines
137 B
Text
Raw Permalink Normal View History

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