mirror of https://github.com/nmvdw/HITs-Examples
Interval is K-finite
This commit is contained in:
parent
8ff54def39
commit
da60017367
|
@ -143,5 +143,16 @@ Section k_properties.
|
|||
- apply (tr loop).
|
||||
- apply path_ishprop.
|
||||
Defined.
|
||||
|
||||
|
||||
Lemma I_Kfinite : Kf interval.
|
||||
Proof.
|
||||
apply Kf_unfold.
|
||||
exists {|Interval.one|}.
|
||||
intro a. simpl.
|
||||
simple refine (interval_ind (fun z => Trunc (-1) (z = Interval.one)) _ _ _ a); simpl.
|
||||
- apply (tr seg).
|
||||
- apply (tr idpath).
|
||||
- apply path_ishprop.
|
||||
Defined.
|
||||
|
||||
End k_properties.
|
||||
|
|
Loading…
Reference in New Issue