src/HOL/Rational.thy
changeset 32069 6d28bbd33e2c
parent 31998 2c7a24f74db9
child 32657 5f13912245ff
equal deleted inserted replaced
32068:98acc234d683 32069:6d28bbd33e2c
  1001   "Fract a b / Fract c d = Fract_norm (a * d) (b * c)"
  1001   "Fract a b / Fract c d = Fract_norm (a * d) (b * c)"
  1002   by simp
  1002   by simp
  1003 
  1003 
  1004 definition (in term_syntax)
  1004 definition (in term_syntax)
  1005   valterm_fract :: "int \<times> (unit \<Rightarrow> Code_Eval.term) \<Rightarrow> int \<times> (unit \<Rightarrow> Code_Eval.term) \<Rightarrow> rat \<times> (unit \<Rightarrow> Code_Eval.term)" where
  1005   valterm_fract :: "int \<times> (unit \<Rightarrow> Code_Eval.term) \<Rightarrow> int \<times> (unit \<Rightarrow> Code_Eval.term) \<Rightarrow> rat \<times> (unit \<Rightarrow> Code_Eval.term)" where
  1006   [code_inline]: "valterm_fract k l = Code_Eval.valtermify Fract {\<cdot>} k {\<cdot>} l"
  1006   [code_unfold]: "valterm_fract k l = Code_Eval.valtermify Fract {\<cdot>} k {\<cdot>} l"
  1007 
  1007 
  1008 notation fcomp (infixl "o>" 60)
  1008 notation fcomp (infixl "o>" 60)
  1009 notation scomp (infixl "o\<rightarrow>" 60)
  1009 notation scomp (infixl "o\<rightarrow>" 60)
  1010 
  1010 
  1011 instantiation rat :: random
  1011 instantiation rat :: random