src/HOL/ex/NormalForm.thy
changeset 21046 fe1db2f991a7
parent 20922 14873e42659c
child 21059 361e62500ab7
equal deleted inserted replaced
21045:66d6d1b0ddfa 21046:fe1db2f991a7
   125  shows "delayed_if True f g = f()" and "delayed_if False f g = g()"
   125  shows "delayed_if True f g = f()" and "delayed_if False f g = g()"
   126 by (auto simp:delayed_if_def)
   126 by (auto simp:delayed_if_def)
   127 
   127 
   128 hide (open) const delayed_if
   128 hide (open) const delayed_if
   129 
   129 
   130 normal_form "OperationalEquality.eq [2..<4] [2,3]"
   130 normal_form "Code_Generator.eq [2..<4] [2,3]"
   131 (*lemma "OperationalEquality.eq [2..<4] [2,3]" by normalization*)
   131 (*lemma "Code_Generator.eq [2..<4] [2,3]" by normalization*)
   132 
   132 
   133 definition
   133 definition
   134  andalso :: "bool \<Rightarrow> bool \<Rightarrow> bool"
   134  andalso :: "bool \<Rightarrow> bool \<Rightarrow> bool"
   135 "andalso x y = (if x then y else False)"
   135 "andalso x y = (if x then y else False)"
   136 
   136