lean2/tests/lean/run/cody1.lean
Leonardo de Moura 70c0eda9fc feat(frontends/lean): make sure all scopes are closed in the end of the module
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2014-08-07 17:08:59 -07:00

25 lines
499 B
Text

import logic
abbreviation subsets (P : Type) := P → Prop.
section
hypothesis A : Type.
hypothesis r : A → subsets A.
hypothesis i : subsets A → A.
hypothesis retract {P : subsets A} {a : A} : r (i P) a = P a.
definition delta (a:A) : Prop := ¬ (r a a).
notation `δ` := delta.
-- Crashes unifier!
theorem false_aux : ¬ (δ (i delta))
:= assume H : δ (i delta),
have H' : r (i delta) (i delta),
from eq_rec H (symm retract),
H H'.
end