mirror of https://github.com/nmvdw/HITs-Examples
Merge branch 'master' of https://github.com/nmvdw/HITs-Examples
This commit is contained in:
commit
39d888951e
|
@ -144,6 +144,17 @@ Section k_properties.
|
|||
- 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.
|
||||
|
||||
Section alternative_definition.
|
||||
|
|
Loading…
Reference in New Issue