1 (**************************************************************************)
4 (* ||A|| A project by Andrea Asperti *)
6 (* ||I|| Developers: *)
7 (* ||T|| The HELM team. *)
8 (* ||A|| http://helm.cs.unibo.it *)
10 (* \ / This file is distributed under the terms of the *)
11 (* v GNU General Public License Version 2 *)
13 (**************************************************************************)
15 include "basics/core_notation.ma".
17 universe constraint Type[0] < Type[1].
18 universe constraint Type[1] < Type[2].
19 universe constraint Type[2] < Type[3].
20 universe constraint Type[3] < Type[4].
22 (*inductive True : Prop ≝ I : True.
24 (*lemma fa : ∀X:Prop.X → X.
32 inductive False : Prop ≝ .
34 inductive bool : Prop ≝ True : bool | false : bool.
36 inductive eq (A:Type[1]) (x:A) : A → Prop ≝
39 lemma provable_True : <A href="cic:/matita/basics/pts/True.ind(1,0,0)">True</A> → eq Prop True True.