src/HOL/Predicate_Compile_Examples/Examples.thy
changeset 52666 391913d17d15
parent 51144 0ede9e2266a8
child 53015 a1119cf551e8
--- a/src/HOL/Predicate_Compile_Examples/Examples.thy	Mon Jul 15 20:13:30 2013 +0200
+++ b/src/HOL/Predicate_Compile_Examples/Examples.thy	Mon Jul 15 20:36:27 2013 +0200
@@ -29,7 +29,8 @@
                          (s1 @ rhs @ s2) = rsl \<and>
                          (rule lhs rhs) \<in> fst g }"
 
-definition derivesp :: "(('nts, 'ts) rule => bool) * 'nts => ('nts, 'ts) symbol list => ('nts, 'ts) symbol list => bool"
+definition derivesp ::
+  "(('nts, 'ts) rule => bool) * 'nts => ('nts, 'ts) symbol list => ('nts, 'ts) symbol list => bool"
 where
   "derivesp g = (\<lambda> lhs rhs. (lhs, rhs) \<in> derives (Collect (fst g), snd g))"
  
@@ -252,7 +253,8 @@
 where
   irconst: "eval_var (IrConst i) conf (IntVal i)"
 | objaddr: "\<lbrakk> Env conf n = i \<rbrakk> \<Longrightarrow> eval_var (ObjAddr n) conf (IntVal i)"
-| plus: "\<lbrakk> eval_var l conf (IntVal vl); eval_var r conf (IntVal vr) \<rbrakk> \<Longrightarrow> eval_var (Add l r) conf (IntVal (vl+vr))"
+| plus: "\<lbrakk> eval_var l conf (IntVal vl); eval_var r conf (IntVal vr) \<rbrakk> \<Longrightarrow>
+    eval_var (Add l r) conf (IntVal (vl+vr))"
 
 
 code_pred eval_var .