faee08591f
This is a big change because we have to store in constraints whether we can use the "relaxed" rules or not. The "relaxed" case says that when type checking the value of an opaque definition we can treat other opaque definitions in the same module as transparent. Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
11 lines
278 B
Text
11 lines
278 B
Text
import standard
|
|
|
|
hypothesis I : Type
|
|
definition F (X : Type) : Type := (X → Prop) → Prop
|
|
hypothesis unfold : I → F I
|
|
hypothesis fold : F I → I
|
|
hypothesis iso1 : ∀x, fold (unfold x) = x
|
|
|
|
variable sorry {A : Type} : A
|
|
theorem iso2 : ∀x, fold (unfold x) = x
|
|
:= sorry
|