X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=helm%2FEXPORT%2Fexportprove%2Fprove%2FprovaIota.v;fp=helm%2FEXPORT%2Fexportprove%2Fprove%2FprovaIota.v;h=0000000000000000000000000000000000000000;hb=e108abe5c0b4eb841c4ad332229a6c0e57e70079;hp=74a510b5dfc84b957939e6bab655d3507094e087;hpb=1456c337a60f6677ee742ff7891d43fc382359a9;p=helm.git diff --git a/helm/EXPORT/exportprove/prove/provaIota.v b/helm/EXPORT/exportprove/prove/provaIota.v deleted file mode 100644 index 74a510b5d..000000000 --- a/helm/EXPORT/exportprove/prove/provaIota.v +++ /dev/null @@ -1,53 +0,0 @@ -Inductive bool : Set := true : bool | false : bool. -Inductive nat : Set := O : nat | S : nat -> nat. - -Fixpoint plus [n:nat] : nat -> nat := - [m:nat] - Cases n of - O => m - | (S n) => (S (plus n m)) - end. - -Fixpoint mult [n:nat] : nat -> nat := - [m:nat] - Cases n of - O => O - | (S n) => (plus m (mult n m)) - end. - -Fixpoint fact [n:nat] : nat := - Cases n of - O => (S O) - | (S n) => (mult (S n) (fact n)) - end. - -Definition bnot := - [b:bool] - Cases b of - true => false - | false => true - end. - -Fixpoint is_even [n:nat] : bool := - Cases n of - O => true - | (S n) => (bnot (bnot (is_odd n))) - end -with is_odd [n:nat] : bool := - Cases n of - O => false - | (S n) => (bnot (bnot (is_even n))) - end -. - -Fixpoint idn [n:nat] : nat := - Cases n of - O => O - | (S n) => (S (idn n)) - end. - -Definition test1 := (is_even (S (S O))). -Definition test2 := (is_even (S (S (S O)))). -Definition test3 := (idn (idn (S O))). -Definition test4 := (is_odd (fact (S (S (O))))). -Definition test5 := (is_odd (fact (S (S (S (S (S (S O)))))))).