changeset 21404 | eb85850d3eb7 |
parent 21378 | cedfce6fc725 |
child 21454 | a1937c51ed88 |
--- a/src/HOL/Code_Generator.thy Fri Nov 17 02:19:55 2006 +0100 +++ b/src/HOL/Code_Generator.thy Fri Nov 17 02:20:03 2006 +0100 @@ -175,7 +175,7 @@ text {* lazy @{const If} *} definition - if_delayed :: "bool \<Rightarrow> (bool \<Rightarrow> 'a) \<Rightarrow> (bool \<Rightarrow> 'a) \<Rightarrow> 'a" + if_delayed :: "bool \<Rightarrow> (bool \<Rightarrow> 'a) \<Rightarrow> (bool \<Rightarrow> 'a) \<Rightarrow> 'a" where "if_delayed b f g = (if b then f True else g False)" lemma [code func]: