Quot/Examples/IntEx.thy
changeset 766 df053507edba
parent 764 a603aa6c9d01
child 767 37285ec4387d
equal deleted inserted replaced
765:d0250d01782c 766:df053507edba
     5 fun
     5 fun
     6   intrel :: "(nat \<times> nat) \<Rightarrow> (nat \<times> nat) \<Rightarrow> bool" (infix "\<approx>" 50)
     6   intrel :: "(nat \<times> nat) \<Rightarrow> (nat \<times> nat) \<Rightarrow> bool" (infix "\<approx>" 50)
     7 where
     7 where
     8   "intrel (x, y) (u, v) = (x + v = u + y)"
     8   "intrel (x, y) (u, v) = (x + v = u + y)"
     9 
     9 
    10 quotient my_int = "nat \<times> nat" / intrel
    10 quotient_type my_int = "nat \<times> nat" / intrel
    11   apply(unfold equivp_def)
    11   apply(unfold equivp_def)
    12   apply(auto simp add: mem_def expand_fun_eq)
    12   apply(auto simp add: mem_def expand_fun_eq)
    13   done
    13   done
    14 
    14 
    15 thm quot_equiv
    15 thm quot_equiv