src/HOL/Imperative_HOL/Heap_Monad.thy
changeset 35423 6ef9525a5727
parent 35113 1a0c129bb2e0
child 36057 ca6610908ae9
--- a/src/HOL/Imperative_HOL/Heap_Monad.thy	Mon Mar 01 17:45:19 2010 +0100
+++ b/src/HOL/Imperative_HOL/Heap_Monad.thy	Mon Mar 01 21:41:35 2010 +0100
@@ -286,14 +286,14 @@
 by auto
 
 lemma graph_implies_dom:
-	"mrec_graph x y \<Longrightarrow> mrec_dom x"
+  "mrec_graph x y \<Longrightarrow> mrec_dom x"
 apply (induct rule:mrec_graph.induct) 
 apply (rule accpI)
 apply (erule mrec_rel.cases)
 by simp
 
 lemma f_default: "\<not> mrec_dom (f, g, x, h) \<Longrightarrow> mrec f g x h = (Inr Exn, undefined)"
-	unfolding mrec_def 
+  unfolding mrec_def 
   by (rule fundef_default_value[OF mrec_sumC_def graph_implies_dom, of _ _ "(f, g, x, h)", simplified])
 
 lemma f_di_reverse: