]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/library/nat/permutation.ma
...
[helm.git] / matita / library / nat / permutation.ma
index 9ab0358c580b231e7d30b0dc41eaeaa9cd87d7b2..768e0bd6091c50c0b4bc93ff767b4820e978c2c3 100644 (file)
@@ -73,7 +73,18 @@ match eqb n i with
       match eqb n j with
       [ true \Rightarrow i
       | false \Rightarrow n]].
-      
+
+notation < "(❲i↹j❳)n"
+  right associative with precedence 71 
+for @{ 'transposition $i $j $n}.
+
+notation < "(❲i \atop j❳)n"
+  right associative with precedence 71 
+for @{ 'transposition $i $j $n}.
+
+interpretation "natural transposition" 'transposition i j n =
+  (cic:/matita/nat/permutation/transpose.con i j n).
+
 lemma transpose_i_j_i: \forall i,j:nat. transpose i j i = j.
 intros.unfold transpose.
 rewrite > (eqb_n_n i).simplify. reflexivity.