]> matita.cs.unibo.it Git - helm.git/commitdiff
letins are no more unfolded, we do that by hand
authorEnrico Tassi <enrico.tassi@inria.fr>
Thu, 20 Mar 2008 12:42:45 +0000 (12:42 +0000)
committerEnrico Tassi <enrico.tassi@inria.fr>
Thu, 20 Mar 2008 12:42:45 +0000 (12:42 +0000)
helm/software/matita/tests/bad_induction.ma

index 172aa8e117a87efc75d3c7a8ab3be7348d701ec2..99c6b5898b6c0680c9c7d3dea3a302cf66066902 100644 (file)
@@ -23,5 +23,5 @@ axiom bad_ind : ∀P : nat -> Prop. ∀n.(n = O -> P n) -> (∀n.P n -> P (S n))
 theorem absurd: ∀n. n = O.
   intros.
   letin P ≝ (λx:nat. n = O).
-  apply (bad_ind P n); simplify; intros; autobatch.
+  apply (bad_ind P n); simplify; intros; unfold; autobatch.
 qed.
\ No newline at end of file