From: Claudio Sacerdoti Coen Date: Mon, 15 Oct 2007 14:01:47 +0000 (+0000) Subject: Dead code clean-up. X-Git-Tag: 0.4.95@7852~113 X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=commitdiff_plain;h=af0e62403bbbc7045efed096261d473da24eb446;p=helm.git Dead code clean-up. --- diff --git a/matita/tests/coercions_propagation.ma b/matita/tests/coercions_propagation.ma index ce8f2e2a7..63c48e66b 100644 --- a/matita/tests/coercions_propagation.ma +++ b/matita/tests/coercions_propagation.ma @@ -16,7 +16,6 @@ set "baseuri" "cic:/matita/test/coercions_propagation/". include "logic/connectives.ma". include "nat/orders.ma". -alias num (instance 0) = "natural number". inductive sigma (A:Type) (P:A → Prop) : Type ≝ sigma_intro: ∀a:A. P a → sigma A P. @@ -33,7 +32,6 @@ definition eject ≝ λP.λc: ∃n:nat.P n. match c with [ sigma_intro w _ ⇒ w coercion cic:/matita/test/coercions_propagation/eject.con. alias num (instance 0) = "natural number". - theorem test: ∃n. 0 ≤ n. apply (S O : ∃n. 0 ≤ n). autobatch.