4 lines
128 B
Text
4 lines
128 B
Text
constants (P : ℕ → Prop) (Q : Prop)
|
||
lemma foo [intro!] [forward] : (: P 0 :) → Q := sorry
|
||
example : P 0 → Q :=
|
||
by grind
|