]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/lib/pts_dummy/CC2FO_K.ma
- pts_dummy/pts_dummy_new: non compiling parts commented out
[helm.git] / matita / matita / lib / pts_dummy / CC2FO_K.ma
index 752ed00c09e009851c1212f1545c50536bc0a9a1..0983db3baafb6089160a48b6c11914172160ad58 100644 (file)
@@ -12,8 +12,8 @@
 (*                                                                        *)
 (**************************************************************************)
 
-include "degree.ma".
-
+include "pts_dummy/degree.ma".
+(*
 (* TO BE PUT ELSEWERE *)
 lemma cons_append_assoc: ∀A,a. ∀l1,l2:list A. (a::l1) @ l2 = a :: (l1 @ l2).
 // qed.
@@ -149,3 +149,4 @@ let rec KI G ≝ match G with
 ].
 
 interpretation "CC2FO: K interpretation (context)" 'IK G = (KI G).
+*)