]> matita.cs.unibo.it Git - helm.git/commitdiff
Spurious code removed.
authorClaudio Sacerdoti Coen <claudio.sacerdoticoen@unibo.it>
Mon, 15 Oct 2007 11:29:04 +0000 (11:29 +0000)
committerClaudio Sacerdoti Coen <claudio.sacerdoticoen@unibo.it>
Mon, 15 Oct 2007 11:29:04 +0000 (11:29 +0000)
Destruct fails recursively.

matita/tests/discriminate.ma

index b1d7b9ca68a74ef5b96959ee19e4ccbe2031cee5..1d6a51494a7faf854732dc965a4ed5666ec9fa6d 100644 (file)
@@ -86,37 +86,11 @@ qed.
 theorem recursive4: ∀ x,y,z,t : nat. 
   C2 ? ? (None ?) ? (S O) ? z (C1 ? ? (S O) (Some ? z) y) = 
   C2 ? ? (None ?) ? (S O) ? t (C1 ? ? (S O) (Some ? x) y) → z=t.
-intros; 
-
-
-
-
- (λHH  : ((C1 (option nat) nat (S O) (Some nat -7) -8) = (C1 (option nat) nat (S O) (Some nat -9) -8))
-  eq_elim_r 
-    (complex (option nat) nat -8 (Some nat -7)) 
-    (C1 (option nat) nat (S O) (Some nat -9) -8) 
-    (λc:(complex (option nat) nat -8 (Some nat -7)).
-      (eq (option nat) 
-        ((λx:(complex (option nat) nat -8 (Some nat -7)).
-           match x return (λy1:nat.(λy2:(option nat).(λ x:(complex (option nat) nat y1 y2).(option nat)))) with
-           [ (C1 (y1:nat) (a:(option nat)) (b:nat)) => a
-           | (C2 (a:(option nat)) (a1:(option nat)) (b:nat) (b1:nat) (y2:nat) (y3:(complex (option nat) nat b1 a1))) ⇒
-              (Some nat -7)
-           ]) c) 
-        (Some nat -9))) 
-     ? 
-     (C1 (option nat) nat (S O) (Some nat -7) -8) 
-     HH)
-
-
-
-
-destruct H;assumption.
+intros; destruct H;assumption.
 qed.
 
 theorem recursive2: ∀ x,y : nat. 
   C2 ? ? (None ?) ? (S O) ? O (C1 ? ? O     (Some ? x) y) = 
   C2 ? ? (None ?) ? (S O) ? O (C1 ? ? (S O) (Some ? x) y) → False.
-intros; destruct H;
-
-
+intros; destruct H.
+qed.
\ No newline at end of file