src/ZF/UNITY/Increasing.thy
changeset 76217 8655344f1cf6
parent 76216 9fc34f76b4e8
child 80917 2a77bc3b4eac
--- a/src/ZF/UNITY/Increasing.thy	Tue Sep 27 17:54:20 2022 +0100
+++ b/src/ZF/UNITY/Increasing.thy	Tue Sep 27 18:02:34 2022 +0100
@@ -48,7 +48,7 @@
 
 lemma increasing_constant [simp]: 
  "F \<in> increasing[A](r, \<lambda>s. c) \<longleftrightarrow> F \<in> program \<and> c \<in> A"
-apply (unfold increasing_def stable_def)
+  unfolding increasing_def stable_def
 apply (subgoal_tac "\<exists>x. x \<in> state")
 apply (auto dest: stable_type [THEN subsetD] intro: st0_in_state)
 done
@@ -94,7 +94,7 @@
 lemma increasing_imp_Increasing: 
      "F \<in> increasing[A](r, f) \<Longrightarrow> F \<in> Increasing[A](r, f)"
 
-apply (unfold increasing_def Increasing_def)
+  unfolding increasing_def Increasing_def
 apply (auto intro: stable_imp_Stable)
 done