src/Doc/Codegen/Computations.thy
changeset 74582 882de99c7c83
parent 69660 2bc2a8599369
child 74584 c14787d73db6
equal deleted inserted replaced
74581:e5b38bb5a147 74582:882de99c7c83
   270 \<close>
   270 \<close>
   271 
   271 
   272 ML %quote \<open>
   272 ML %quote \<open>
   273   local
   273   local
   274 
   274 
   275   fun raw_dvd (b, ct) = Thm.mk_binop \<^cterm>\<open>Pure.eq :: bool \<Rightarrow> bool \<Rightarrow> prop\<close>
   275   fun raw_dvd (b, ct) =
   276     ct (if b then \<^cterm>\<open>True\<close> else \<^cterm>\<open>False\<close>);
   276     \<^instantiate>\<open>x = ct and y = \<open>if b then \<^cterm>\<open>True\<close> else \<^cterm>\<open>False\<close>\<close>
       
   277       in cterm "x \<equiv> y" for x y :: bool\<close>;
   277 
   278 
   278   val (_, dvd_oracle) = Context.>>> (Context.map_theory_result
   279   val (_, dvd_oracle) = Context.>>> (Context.map_theory_result
   279     (Thm.add_oracle (\<^binding>\<open>dvd\<close>, raw_dvd)));
   280     (Thm.add_oracle (\<^binding>\<open>dvd\<close>, raw_dvd)));
   280 
   281 
   281   in
   282   in