2014-08-24 19:58:48 -07:00
|
|
|
import logic
|
2014-07-27 12:01:06 -07:00
|
|
|
|
2014-10-02 16:20:52 -07:00
|
|
|
axiom I : Type
|
2014-07-27 12:01:06 -07:00
|
|
|
definition F (X : Type) : Type := (X → Prop) → Prop
|
2014-10-02 16:20:52 -07:00
|
|
|
axiom unfold : I → F I
|
2015-03-25 18:22:20 -07:00
|
|
|
axiom foldd : F I → I
|
|
|
|
axiom iso1 : ∀x, foldd (unfold x) = x
|
2014-07-27 12:01:06 -07:00
|
|
|
|
2015-03-25 18:22:20 -07:00
|
|
|
theorem iso2 : ∀x, foldd (unfold x) = x
|
2014-07-27 12:01:06 -07:00
|
|
|
:= sorry
|