lean2/tests/lean/red.lean
Leonardo de Moura 11aad4449b feat(frontends/lean): add '[semireducible]' attribute
This commit also renames the elements of reducible_status.
The idea is to use in the C++ implementation the same names used in the
Lean front-end.
2015-03-03 10:48:36 -08:00

26 lines
432 B
Text

constant g : nat → nat
definition f := g
example : f = g := rfl
attribute f [irreducible]
example : f = g := rfl -- Error
example (a : nat) (H : a = g a) : f a = a :=
eq.subst H rfl -- Error
attribute f [semireducible]
example (a : nat) (H : a = g a) : f a = a :=
eq.subst H rfl -- Error
example : f = g := rfl
attribute f [reducible]
example : f = g := rfl
example (a : nat) (H : a = g a) : f a = a :=
eq.subst H rfl