]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/contribs/dama/dama/bishop_set.ma
initial qork for models
[helm.git] / helm / software / matita / contribs / dama / dama / bishop_set.ma
index 1e7436af9a3e97d347a47dc259c726537e2a06be..d572820799b26ed2080451ef81083c0064784a86 100644 (file)
@@ -23,11 +23,10 @@ record bishop_set: Type ≝ {
   bs_cotransitive: cotransitive ? bs_apart
 }.
 
-notation "hvbox(a break # b)" non associative with precedence 50 
+notation "hvbox(a break # b)" non associative with precedence 45 
   for @{ 'apart $a $b}.
   
-interpretation "bishop_setapartness" 'apart x y = 
-  (cic:/matita/dama/bishop_set/bs_apart.con _ x y).
+interpretation "bishop_setapartness" 'apart x y = (bs_apart _ x y).
 
 definition bishop_set_of_ordered_set: ordered_set → bishop_set.
 intros (E); apply (mk_bishop_set E (λa,b:E. a ≰ b ∨ b ≰ a));  
@@ -42,11 +41,10 @@ qed.
 (* Definition 2.2 (2) *)
 definition eq ≝ λA:bishop_set.λa,b:A. ¬ (a # b).
 
-notation "hvbox(a break ≈ b)" non associative with precedence 50 
+notation "hvbox(a break ≈ b)" non associative with precedence 45 
   for @{ 'napart $a $b}.
       
-interpretation "Bishop set alikeness" 'napart a b = 
-  (cic:/matita/dama/bishop_set/eq.con _ a b). 
+interpretation "Bishop set alikeness" 'napart a b = (eq _ a b). 
 
 lemma eq_reflexive:∀E:bishop_set. reflexive ? (eq E).
 intros (E); unfold; intros (x); apply bs_coreflexive; 
@@ -78,8 +76,7 @@ qed.
 
 definition lt ≝ λE:ordered_set.λa,b:E. a ≤ b ∧ a # b.
 
-interpretation "ordered sets less than" 'lt a b = 
-  (cic:/matita/dama/bishop_set/lt.con _ a b).
+interpretation "ordered sets less than" 'lt a b = (lt _ a b).
 
 lemma lt_coreflexive: ∀E.coreflexive ? (lt E).
 intros 2 (E x); intro H; cases H (_ ABS);