lean2/tests/lean/omit.lean
2014-10-09 07:13:06 -07:00

22 lines
285 B
Text

section
variable A : Type
variable a : A
variable c : A
omit A
include A
include A
omit A
variable B : Type
variable b : B
variable d : B
include A
include a
include c
definition foo := b
inductive tst (C : Type) :=
mk : tst C
end
check foo
check tst