]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/tests/bad_induction.ma
updating the structures for sorts
[helm.git] / helm / software / matita / tests / bad_induction.ma
index b009e18d15d04aea4302428a440804967931a580..99c6b5898b6c0680c9c7d3dea3a302cf66066902 100644 (file)
@@ -12,7 +12,7 @@
 (*                                                                        *)
 (**************************************************************************)
 
-set "baseuri" "cic:/matita/nat/bad_induction".
+
 
 include "nat/nat.ma".
 
@@ -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