From af0e62403bbbc7045efed096261d473da24eb446 Mon Sep 17 00:00:00 2001 From: Claudio Sacerdoti Coen Date: Mon, 15 Oct 2007 14:01:47 +0000 Subject: [PATCH] Dead code clean-up. --- matita/tests/coercions_propagation.ma | 2 -- 1 file changed, 2 deletions(-) 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. -- 2.39.2