]> matita.cs.unibo.it Git - helm.git/blobdiff - weblib/basics/pts.ma
commit by user andrea
[helm.git] / weblib / basics / pts.ma
index 1b87a2d0b18e1dc2d5e16d228f4a9d5bf78fc79e..b7d9a5da9deb592e73670182de1459befd569321 100644 (file)
@@ -19,23 +19,3 @@ 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