]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/matita/tests/inversion.ma
various updates, removed proofs for now because they are the real bottleneck!!
[helm.git] / helm / matita / tests / inversion.ma
index ccbc4d96b7f2e85b56ecc628f4deb8a9094b5dc0..5f173344454084a0f2fd296b9732d4ba2f16729c 100644 (file)
@@ -1,3 +1,5 @@
+set "baseuri" "cic:/matita/tests/".
+
 inductive nat : Set \def
    O : nat
  | S : nat \to nat.
@@ -18,5 +20,5 @@ theorem test_inversion: \forall n. le n O \to n=O.
   apply (le_ind ? (\lambda x. O=x \to n=x) ? ? ? H).
   intro. reflexivity.
   simplify. intros.
-  (* manca discriminate H3 *)
-qed.
\ No newline at end of file
+  discriminate H3.
+qed.