src/HOL/Real.thy
changeset 72581 de581f98a3a1
parent 72569 d56e4eeae967
child 72607 feebdaa346e5
equal deleted inserted replaced
72580:531a0c44ea3f 72581:de581f98a3a1
  1636 
  1636 
  1637 definition (in term_syntax)
  1637 definition (in term_syntax)
  1638   valterm_ratreal :: "rat \<times> (unit \<Rightarrow> Code_Evaluation.term) \<Rightarrow> real \<times> (unit \<Rightarrow> Code_Evaluation.term)"
  1638   valterm_ratreal :: "rat \<times> (unit \<Rightarrow> Code_Evaluation.term) \<Rightarrow> real \<times> (unit \<Rightarrow> Code_Evaluation.term)"
  1639   where [code_unfold]: "valterm_ratreal k = Code_Evaluation.valtermify Ratreal {\<cdot>} k"
  1639   where [code_unfold]: "valterm_ratreal k = Code_Evaluation.valtermify Ratreal {\<cdot>} k"
  1640 
  1640 
  1641 notation fcomp (infixl "\<circ>>" 60)
       
  1642 notation scomp (infixl "\<circ>\<rightarrow>" 60)
       
  1643 
       
  1644 instantiation real :: random
  1641 instantiation real :: random
  1645 begin
  1642 begin
  1646 
  1643 
       
  1644 context
       
  1645   includes state_combinator_syntax
       
  1646 begin
       
  1647 
  1647 definition
  1648 definition
  1648   "Quickcheck_Random.random i = Quickcheck_Random.random i \<circ>\<rightarrow> (\<lambda>r. Pair (valterm_ratreal r))"
  1649   "Quickcheck_Random.random i = Quickcheck_Random.random i \<circ>\<rightarrow> (\<lambda>r. Pair (valterm_ratreal r))"
  1649 
  1650 
  1650 instance ..
  1651 instance ..
  1651 
  1652 
  1652 end
  1653 end
  1653 
  1654 
  1654 no_notation fcomp (infixl "\<circ>>" 60)
  1655 end
  1655 no_notation scomp (infixl "\<circ>\<rightarrow>" 60)
       
  1656 
  1656 
  1657 instantiation real :: exhaustive
  1657 instantiation real :: exhaustive
  1658 begin
  1658 begin
  1659 
  1659 
  1660 definition
  1660 definition