]> matita.cs.unibo.it Git - helm.git/blobdiff - weblib/basics/pts.ma
grafite parser updated
[helm.git] / weblib / basics / pts.ma
index 1b87a2d0b18e1dc2d5e16d228f4a9d5bf78fc79e..c0ec34b71cf9d3a0d431a8153ad033ada3fcd67a 100644 (file)
@@ -18,24 +18,5 @@ universe constraint Type[0] < Type[1].
 universe constraint Type[1] < Type[2].
 universe constraint Type[2] < Type[3].
 universe constraint Type[3] < Type[4].
-
-(*inductive True : Prop ≝ I : True.
-
-(*lemma fa : ∀X:Prop.X → X.
-#X #p //
-qed.
-
-(* check fa*)
-
-lemma ggr ≝ fa.*)
-
-inductive False : Prop ≝ .
-
-inductive bool : Prop ≝ True : bool | false : bool.
-inductive eq (A:Type[1]) (x:A) : A → Prop ≝
-    refl: eq A x x.
-
-lemma provable_True : <A href="cic:/matita/basics/pts/True.ind(1,0,0)">True</A> → eq Prop True True.
-#H %
-qed.*)
\ No newline at end of file
+universe constraint Type[4] < Type[5].
\ No newline at end of file