lean2/tests/lean/run/simplifier1.lean

12 lines
263 B
Text
Raw Normal View History

constant P : Type₁
constant P_sub : subsingleton P
attribute P_sub [instance]
constant q : P → nat → Prop
set_option blast.simp false
2015-12-09 04:06:43 +00:00
set_option trace.blast true
set_option trace.cc true
example (a : nat) (h₁ h₂ : P) : q h₁ a = q h₂ a :=
by blast