2015-12-03 22:21:30 +00:00
|
|
|
constant P : Type₁
|
|
|
|
constant P_sub : subsingleton P
|
|
|
|
attribute P_sub [instance]
|
|
|
|
constant q : P → Prop
|
|
|
|
|
|
|
|
section
|
|
|
|
example (h₁ h₂ : P) : q h₁ = q h₂ :=
|
2015-12-06 23:01:49 +00:00
|
|
|
by simp
|
2015-12-03 22:21:30 +00:00
|
|
|
end
|
|
|
|
|
|
|
|
|
|
|
|
section
|
2015-12-06 23:01:49 +00:00
|
|
|
set_option blast.strategy "cc"
|
2015-12-03 22:21:30 +00:00
|
|
|
|
|
|
|
example (h₁ h₂ : P) : q h₁ = q h₂ :=
|
|
|
|
by blast
|
|
|
|
end
|