]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/contribs/ng_TPTP/COL029-1.ma
tacticals are really tactics now, they have an AST at the same level of
[helm.git] / helm / software / matita / contribs / ng_TPTP / COL029-1.ma
index 7247922708b8e920eb333fdd8e3ff8ce70863052..2b8dd1498f124c9876407a6c0cd787a9c4ca9669 100644 (file)
@@ -54,24 +54,23 @@ include "logic/equality.ma".
 
 (* -------------------------------------------------------------------------- *)
 ntheorem prove_fixed_point:
- ∀Univ:Type.∀X:Univ.∀Y:Univ.
(∀Univ:Type.∀X:Univ.∀Y:Univ.
 ∀apply:∀_:Univ.∀_:Univ.Univ.
 ∀f:∀_:Univ.Univ.
 ∀u:Univ.
-∀H0:∀X:Univ.∀Y:Univ.eq Univ (apply (apply u X) Y) (apply Y (apply (apply X X) Y)).∃Y:Univ.eq Univ (apply Y (f Y)) (apply (f Y) (apply Y (f Y)))
+∀H0:∀X:Univ.∀Y:Univ.eq Univ (apply (apply u X) Y) (apply Y (apply (apply X X) Y)).∃Y:Univ.eq Univ (apply Y (f Y)) (apply (f Y) (apply Y (f Y))))
 .
-#Univ.
-#X.
-#Y.
-#apply.
-#f.
-#u.
-#H0.
-napply ex_intro[
-nid2:
-nauto by H0;
-nid|
-skip]
+#Univ ##.
+#X ##.
+#Y ##.
+#apply ##.
+#f ##.
+#u ##.
+#H0 ##.
+napply (ex_intro ? ? ? ?) ##[
+##2:
+nauto by H0 ##;
+##| ##skip ##]
 nqed.
 
 (* -------------------------------------------------------------------------- *)