]> matita.cs.unibo.it Git - helm.git/commitdiff
Dead code clean-up.
authorClaudio Sacerdoti Coen <claudio.sacerdoticoen@unibo.it>
Mon, 15 Oct 2007 14:01:47 +0000 (14:01 +0000)
committerClaudio Sacerdoti Coen <claudio.sacerdoticoen@unibo.it>
Mon, 15 Oct 2007 14:01:47 +0000 (14:01 +0000)
matita/tests/coercions_propagation.ma

index ce8f2e2a7af943c4ef1ba0520bd45b5cd732a295..63c48e66b9d42267b3d3455cc855565b80527095 100644 (file)
@@ -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.