lean2/tests/lean/ind_parser_bug.lean
Leonardo de Moura 8723f5b613 fix(frontends/lean/inductive_cmd): inductive datatype elaborator was 'fixing' parameter mismatches.
Given a datatype C with parameters As, if the declaration contained
(C Bs), the elaborator would silently replace it with (C As).

This bug would confuse users and make them believe they define something
different.
2014-11-05 23:12:00 -08:00

15 lines
331 B
Text

import logic
inductive acc1 (A : Type) (R : A → A → Prop) (a : A) : Prop :=
intro : ∀ (x : A), (∀ (y : A), R y x → acc1 A R y) → acc1 A R x
section
variables (A : Type) (R : A → A → Prop)
inductive acc2 (a : A) : Prop :=
intro : ∀ (x : A), (∀ (y : A), R y x → acc2 y) → acc2 x
end
print "done"