]> matita.cs.unibo.it Git - helm.git/commitdiff
Improved tests (for left parameters and mutual recursive definitions).
authorClaudio Sacerdoti Coen <claudio.sacerdoticoen@unibo.it>
Fri, 8 May 2009 21:06:29 +0000 (21:06 +0000)
committerClaudio Sacerdoti Coen <claudio.sacerdoticoen@unibo.it>
Fri, 8 May 2009 21:06:29 +0000 (21:06 +0000)
helm/software/matita/tests/ng_commands.ma

index f816b36840c2b4684593e011fbf8c430c74433d1..755921938d15cb7b6113b2885606fe5a9c1413c8 100644 (file)
@@ -39,23 +39,22 @@ ntheorem nzero_ok: nzero (S (S O)) = O.
  napply (refl_eq ? O);
 nqed.
 
-ninductive nnat: Type ≝
-   nO: nnat
- | nS: mat → mat → nnat
+naxiom DT: nat → Type.
+naxiom dt: ∀n. DT n.
+
+ninductive nnat (n: nat) (A:DT n): Type ≝
+   nO: nnat n A
+ | nS: mat n A → mat n A → nnat n A
 with mat: Type ≝ 
- |mS : nnat → mat
-.
+ |mS : nnat n A → mat n A.
 
-nlet rec nnzero (n:nnat) : nnat ≝
+nlet rec nnzero (n:nnat 0 (dt ?)) : nnat 0 (dt ?) ≝
  match n return ? with
-  [ nO ⇒ nO
+  [ nO ⇒ nO 0 (dt ?)
   | nS m _ ⇒ nmzero m ]
-and nmzero (m:mat) : nnat ≝ 
+and nmzero (m:mat 0 (dt ?)) : nnat 0 (dt ?) ≝ 
  match m return ? with
- [ mS n ⇒ nnzero n ].   
-
-(* testare anche i record e le ricorsioni/coricorsioni/(co)induttivi MUTUI *)
+ [ mS n ⇒ nnzero n ].
 
-(*
-nrecord pair: Type ≝ { l: pair; r: pair }.
-*)
\ No newline at end of file
+nrecord pair (n: nat) (x: dt n) (label: Type): Type ≝
+ { lbl:label; l: pair label; r: pair label}.
\ No newline at end of file