Library mxx
Links: Index_v Table of contents Main page
| P | F | S |
mE |<--:-->: |
mS | :<--:-->|
Inductive Version :=
| vP (* paper *)
| vF (* full *)
| vS (* soundness *)
.
Definition Mode := (bool × Version)%type.
| vP (* paper *)
| vF (* full *)
| vS (* soundness *)
.
Definition Mode := (bool × Version)%type.
The condition mE v is used for premises of P not used in S.
These premises are thus available in both P and E and necessary
for extraction.
Definition mS (v : Mode) :=
match snd v with
| vP ⇒ False
| vF ⇒ True
| vS ⇒ True
end.
Definition mR (v : Mode) :=
match fst v with
| true ⇒ True
| false ⇒ False
end.
Hint Unfold Mode mE mS mR.
match snd v with
| vP ⇒ False
| vF ⇒ True
| vS ⇒ True
end.
Definition mR (v : Mode) :=
match fst v with
| true ⇒ True
| false ⇒ False
end.
Hint Unfold Mode mE mS mR.