4 lines
137 B
Text
4 lines
137 B
Text
import logic.cast
|
|
|
|
theorem cast_heq : ∀ {A B : Type} (H : A = B) (a : A), cast H a == a
|
|
| A A (eq.refl A) a := heq.of_eq (cast_refl a)
|