]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambda_delta/basic_2/grammar/term_simple.ma
- intermediate commit to allow debugging of auto tactic in xprs.ma
[helm.git] / matita / matita / contribs / lambda_delta / basic_2 / grammar / term_simple.ma
index 4c02d521d248770e2546c13dd834b2d608894da2..83aff07c497541a142bbfaabfbb04fdbcd11cc86 100644 (file)
@@ -39,3 +39,8 @@ lemma simple_inv_pair: ∀I,V,T.  𝐒⦃②{I}V.T⦄ → ∃J. I = Flat2 J.
 * /2 width=2/ #I #V #T #H
 elim (simple_inv_bind … H)
 qed-.
+
+(*
+lemma mt: ∀R1,R2:Prop. (R1 → R2) → (R2 → ⊥) → R1 → ⊥.
+/3 width=1/ qed-.
+*)