Require Import TestSuite.admit.
Module NonPrim.
Unset Primitive Projections.
Record hProp := hp { hproptype :> Type }.
Goal forall (h : (Type -> hProp) -> (Type -> hProp)) k f,
(forall y, h y = y) ->
h (fun b : Type => {| hproptype := f b |}) = k.
Proof.
intros h k f H.
etransitivity.
apply H.
admit.
Defined.
End NonPrim.
Module Prim.
Set Primitive Projections.
Record hProp := hp { hproptype :> Type }.
Goal forall (h : (Type -> hProp) -> (Type -> hProp)) k f,
(forall y, h y = y) ->
h (fun b : Type => {| hproptype := f b |}) = k.
Proof.
intros h k f H.
etransitivity.
apply H.
Abort.
End Prim.
¤ Dauer der Verarbeitung: 0.23 Sekunden
(vorverarbeitet)
¤
|
Haftungshinweis
Die Informationen auf dieser Webseite wurden
nach bestem Wissen sorgfältig zusammengestellt. Es wird jedoch weder Vollständigkeit, noch Richtigkeit,
noch Qualität der bereit gestellten Informationen zugesichert.
Bemerkung:
Die farbliche Syntaxdarstellung ist noch experimentell.
|