IntEx2.thy
changeset 581 2da4fb1894d2
parent 579 eac2662a21ec
parent 578 070161f1996a
child 584 97f6e5c61f03
equal deleted inserted replaced
580:fc48fe9667f2 581:2da4fb1894d2
     3 uses
     3 uses
     4   ("Tools/numeral.ML")
     4   ("Tools/numeral.ML")
     5   ("Tools/numeral_syntax.ML")
     5   ("Tools/numeral_syntax.ML")
     6   ("Tools/int_arith.ML")
     6   ("Tools/int_arith.ML")
     7 begin
     7 begin
       
     8 
     8 
     9 
     9 fun
    10 fun
    10   intrel :: "(nat \<times> nat) \<Rightarrow> (nat \<times> nat) \<Rightarrow> bool" (infix "\<approx>" 50)
    11   intrel :: "(nat \<times> nat) \<Rightarrow> (nat \<times> nat) \<Rightarrow> bool" (infix "\<approx>" 50)
    11 where
    12 where
    12   "intrel (x, y) (u, v) = (x + v = u + y)"
    13   "intrel (x, y) (u, v) = (x + v = u + y)"