]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/library/datatypes/subsets.ma
nasty change in the lexer/parser:
[helm.git] / helm / software / matita / library / datatypes / subsets.ma
index 8c7963d67ea3a28b3073cadb844f27d1d25f713a..8e2eda4c99508749053bc3041154e814cdf27fd6 100644 (file)
@@ -59,7 +59,7 @@ definition mem: ∀A. binary_morphism1 A (Ω \sup A) CPROP.
      | apply s1; assumption]]
 qed.     
 
-interpretation "mem" 'mem a S = (fun1 ___ (mem _) a S).
+interpretation "mem" 'mem a S = (fun1 ??? (mem ?) a S).
 
 definition subseteq: ∀A. binary_morphism1 (Ω \sup A) (Ω \sup A) CPROP.
  intros;
@@ -74,7 +74,7 @@ definition subseteq: ∀A. binary_morphism1 (Ω \sup A) (Ω \sup A) CPROP.
       apply (transitive_subseteq_operator ???? s s4) ]]
 qed.
 
-interpretation "subseteq" 'subseteq U V = (fun1 ___ (subseteq _) U V).
+interpretation "subseteq" 'subseteq U V = (fun1 ??? (subseteq ?) U V).
 
 theorem subseteq_refl: ∀A.∀S:Ω \sup A.S ⊆ S.
  intros 4; assumption.
@@ -96,7 +96,7 @@ definition overlaps: ∀A. binary_morphism1 (Ω \sup A) (Ω \sup A) CPROP.
      | apply (. #‡(H1 \sup -1)); assumption]]
 qed.
 
-interpretation "overlaps" 'overlaps U V = (fun1 ___ (overlaps _) U V).
+interpretation "overlaps" 'overlaps U V = (fun1 ??? (overlaps ?) U V).
 
 definition intersects:
  ∀A. binary_morphism1 (powerset_setoid A) (powerset_setoid A) (powerset_setoid A).
@@ -110,7 +110,7 @@ definition intersects:
     | apply (. (#‡(H \sup -1))‡(#‡(H1 \sup -1))); assumption]]
 qed.
 
-interpretation "intersects" 'intersects U V = (fun1 ___ (intersects _) U V).
+interpretation "intersects" 'intersects U V = (fun1 ??? (intersects ?) U V).
 
 definition union:
  ∀A. binary_morphism1 (powerset_setoid A) (powerset_setoid A) (powerset_setoid A).
@@ -124,7 +124,7 @@ definition union:
     | apply (. (#‡(H \sup -1))‡(#‡(H1 \sup -1))); assumption]]
 qed.
 
-interpretation "union" 'union U V = (fun1 ___ (union _) U V).
+interpretation "union" 'union U V = (fun1 ??? (union ?) U V).
 
 definition singleton: ∀A:setoid. unary_morphism A (Ω \sup A).
  intros; constructor 1;
@@ -137,6 +137,6 @@ definition singleton: ∀A:setoid. unary_morphism A (Ω \sup A).
      [ apply a |4: apply a'] try assumption; apply sym; assumption]
 qed.
 
-interpretation "singleton" 'singl a = (fun_1 __ (singleton _) a).
+interpretation "singleton" 'singl a = (fun_1 ?? (singleton ?) a).
 
 *)
\ No newline at end of file